File tree Expand file tree Collapse file tree 1 file changed +2
-6
lines changed
src/Algebra/Properties/Monoid Expand file tree Collapse file tree 1 file changed +2
-6
lines changed Original file line number Diff line number Diff line change @@ -14,17 +14,13 @@ module Algebra.Properties.Monoid.Reasoning {o ℓ} (M : Monoid o ℓ) where
1414
1515open Monoid M
1616 using (Carrier; _∙_; _≈_; setoid; isMagma; semigroup; ε; sym; identityˡ; identityʳ
17- ; ∙-cong; refl; assoc)
17+ ; ∙-cong; refl; assoc; ∙-congˡ; ∙-congʳ )
1818open import Relation.Binary.Reasoning.Setoid setoid
1919open import Algebra.Properties.Semigroup.Reasoning semigroup public
20- open IsMagma isMagma using (∙-congˡ; ∙-congʳ)
2120
2221module Identity {a : Carrier } where
2322 id-unique : (∀ b → b ∙ a ≈ b) → a ≈ ε
24- id-unique b∙a≈b = begin
25- a ≈⟨ sym (identityˡ a) ⟩
26- ε ∙ a ≈⟨ b∙a≈b ε ⟩
27- ε ∎
23+ id-unique b∙a≈b = trans (sym (identityˡ a) ) (b∙a≈b ε)
2824
2925 id-comm : a ∙ ε ≈ ε ∙ a
3026 id-comm = begin
You can’t perform that action at this time.
0 commit comments