Skip to content

Commit fbc01da

Browse files
committed
move importation
1 parent 92b278b commit fbc01da

File tree

1 file changed

+3
-2
lines changed

1 file changed

+3
-2
lines changed

src/Algebra/Properties/Monoid/Reasoning.agda

+3-2
Original file line numberDiff line numberDiff line change
@@ -8,10 +8,11 @@
88
{-# OPTIONS --cubical-compatible --safe #-}
99

1010
open import Algebra.Bundles using (Monoid)
11-
open import Algebra.Structures using (IsMagma)
1211

1312
module Algebra.Properties.Monoid.Reasoning {o ℓ} (M : Monoid o ℓ) where
1413

14+
open import Algebra.Structures using (IsMagma)
15+
1516
open Monoid M
1617
using (Carrier; _∙_; _≈_; setoid; isMagma; semigroup; ε; sym; identityˡ
1718
; identityʳ ; ∙-cong; refl; assoc; ∙-congˡ; ∙-congʳ; trans)
@@ -50,7 +51,7 @@ open IntroElim public
5051

5152
module Cancellers {a b c : Carrier} (inv : a ∙ c ≈ ε) where
5253

53-
cancelʳ : (b ∙ a) ∙ c ≈ b
54+
cancelʳ : (b ∙ a) ∙ c ≈ b
5455
cancelʳ = trans (assoc b a c) (trans (∙-congˡ inv) (identityʳ b))
5556

5657
cancelˡ : a ∙ (c ∙ b) ≈ b

0 commit comments

Comments
 (0)