File tree Expand file tree Collapse file tree 2 files changed +5
-5
lines changed Expand file tree Collapse file tree 2 files changed +5
-5
lines changed Original file line number Diff line number Diff line change 7
7
{-# OPTIONS --cubical-compatible --safe #-}
8
8
9
9
open import Algebra.Bundles using (RawMonoid)
10
- open import Data.Nat.Base as ℕ using (ℕ; zero; suc)
11
- open import Data.Vec.Functional as Vector using (Vector)
12
10
13
11
module Algebra.Definitions.RawMonoid {a ℓ} (M : RawMonoid a ℓ) where
14
12
13
+ open import Data.Nat.Base as ℕ using (ℕ; zero; suc)
14
+ open import Data.Vec.Functional as Vector using (Vector)
15
15
open RawMonoid M renaming ( _∙_ to _+_ ; ε to 0# )
16
16
17
17
------------------------------------------------------------------------
Original file line number Diff line number Diff line change 7
7
{-# OPTIONS --cubical-compatible --safe #-}
8
8
9
9
open import Algebra.Bundles using (RawSemiring)
10
+
11
+ module Algebra.Definitions.RawSemiring {a ℓ} (M : RawSemiring a ℓ) where
12
+
10
13
open import Data.Sum.Base using (_⊎_)
11
14
open import Data.Nat.Base using (ℕ; zero; suc)
12
15
open import Level using (_⊔_)
13
16
open import Relation.Binary.Core using (Rel)
14
-
15
- module Algebra.Definitions.RawSemiring {a ℓ} (M : RawSemiring a ℓ) where
16
-
17
17
open RawSemiring M renaming (Carrier to A)
18
18
19
19
------------------------------------------------------------------------
You can’t perform that action at this time.
0 commit comments