We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 3cbb91b commit 29b22d6Copy full SHA for 29b22d6
src/Algebra/Properties/Monoid/Reasoning.agda
@@ -11,6 +11,8 @@ open import Algebra.Bundles using (Monoid)
11
12
module Algebra.Properties.Monoid.Reasoning {o ℓ} (M : Monoid o ℓ) where
13
14
+open import Algebra.Structures using (IsMagma)
15
+
16
open Monoid M
17
using (Carrier; _∙_; _≈_; setoid; isMagma; semigroup; ε; sym; identityˡ
18
; identityʳ ; ∙-cong; refl; assoc; ∙-congˡ; ∙-congʳ; trans)
@@ -49,7 +51,7 @@ open IntroElim public
49
51
50
52
module Cancellers {a b c : Carrier} (inv : a ∙ c ≈ ε) where
53
- cancelʳ : (b ∙ a) ∙ c ≈ b
54
+ cancelʳ : (b ∙ a) ∙ c ≈ b
55
cancelʳ = trans (assoc b a c) (trans (∙-congˡ inv) (identityʳ b))
56
57
cancelˡ : a ∙ (c ∙ b) ≈ b
0 commit comments