File tree Expand file tree Collapse file tree 1 file changed +3
-2
lines changed
src/Algebra/Properties/Monoid Expand file tree Collapse file tree 1 file changed +3
-2
lines changed Original file line number Diff line number Diff line change 88{-# OPTIONS --cubical-compatible --safe #-}
99
1010open import Algebra.Bundles using (Monoid)
11- open import Algebra.Structures using (IsMagma)
1211
1312module Algebra.Properties.Monoid.Reasoning {o ℓ} (M : Monoid o ℓ) where
1413
14+ open import Algebra.Structures using (IsMagma)
15+
1516open 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
5152module 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
You can’t perform that action at this time.
0 commit comments