Skip to content

Commit 021b69c

Browse files
authored
alegbra.definitions (#2601)
1 parent 68b2bbf commit 021b69c

File tree

2 files changed

+5
-5
lines changed

2 files changed

+5
-5
lines changed

src/Algebra/Definitions/RawMonoid.agda

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -7,11 +7,11 @@
77
{-# OPTIONS --cubical-compatible --safe #-}
88

99
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)
1210

1311
module 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)
1515
open RawMonoid M renaming ( _∙_ to _+_ ; ε to 0# )
1616

1717
------------------------------------------------------------------------

src/Algebra/Definitions/RawSemiring.agda

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -7,13 +7,13 @@
77
{-# OPTIONS --cubical-compatible --safe #-}
88

99
open import Algebra.Bundles using (RawSemiring)
10+
11+
module Algebra.Definitions.RawSemiring {a ℓ} (M : RawSemiring a ℓ) where
12+
1013
open import Data.Sum.Base using (_⊎_)
1114
open import Data.Nat.Base using (ℕ; zero; suc)
1215
open import Level using (_⊔_)
1316
open import Relation.Binary.Core using (Rel)
14-
15-
module Algebra.Definitions.RawSemiring {a ℓ} (M : RawSemiring a ℓ) where
16-
1717
open RawSemiring M renaming (Carrier to A)
1818

1919
------------------------------------------------------------------------

0 commit comments

Comments
 (0)