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 77{-# OPTIONS --cubical-compatible --safe #-}
88
99open 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)
1210
1311module Algebra.Definitions.RawMonoid {a ℓ} (M : RawMonoid a ℓ) where
1412
13+ open import Data.Nat.Base as ℕ using (ℕ; zero; suc)
14+ open import Data.Vec.Functional as Vector using (Vector)
1515open RawMonoid M renaming ( _∙_ to _+_ ; ε to 0# )
1616
1717------------------------------------------------------------------------
Original file line number Diff line number Diff line change 77{-# OPTIONS --cubical-compatible --safe #-}
88
99open import Algebra.Bundles using (RawSemiring)
10+
11+ module Algebra.Definitions.RawSemiring {a ℓ} (M : RawSemiring a ℓ) where
12+
1013open import Data.Sum.Base using (_⊎_)
1114open import Data.Nat.Base using (ℕ; zero; suc)
1215open import Level using (_⊔_)
1316open import Relation.Binary.Core using (Rel)
14-
15- module Algebra.Definitions.RawSemiring {a ℓ} (M : RawSemiring a ℓ) where
16-
1717open RawSemiring M renaming (Carrier to A)
1818
1919------------------------------------------------------------------------
You can’t perform that action at this time.
0 commit comments