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 8
8
{-# OPTIONS --cubical-compatible --safe #-}
9
9
10
10
open import Algebra.Bundles using (Monoid)
11
- open import Algebra.Structures using (IsMagma)
12
11
13
12
module Algebra.Properties.Monoid.Reasoning {o ℓ} (M : Monoid o ℓ) where
14
13
14
+ open import Algebra.Structures using (IsMagma)
15
+
15
16
open Monoid M
16
17
using (Carrier; _∙_; _≈_; setoid; isMagma; semigroup; ε; sym; identityˡ
17
18
; identityʳ ; ∙-cong; refl; assoc; ∙-congˡ; ∙-congʳ; trans)
@@ -50,7 +51,7 @@ open IntroElim public
50
51
51
52
module Cancellers {a b c : Carrier} (inv : a ∙ c ≈ ε) where
52
53
53
- cancelʳ : (b ∙ a) ∙ c ≈ b
54
+ cancelʳ : (b ∙ a) ∙ c ≈ b
54
55
cancelʳ = trans (assoc b a c) (trans (∙-congˡ inv) (identityʳ b))
55
56
56
57
cancelˡ : a ∙ (c ∙ b) ≈ b
You can’t perform that action at this time.
0 commit comments