Skip to content

Commit 5db9ac8

Browse files
committed
fix-whitespace
1 parent fbc01da commit 5db9ac8

File tree

1 file changed

+1
-3
lines changed

1 file changed

+1
-3
lines changed

src/Algebra/Properties/Monoid/Reasoning.agda

+1-3
Original file line numberDiff line numberDiff line change
@@ -11,8 +11,6 @@ open import Algebra.Bundles using (Monoid)
1111

1212
module Algebra.Properties.Monoid.Reasoning {o ℓ} (M : Monoid o ℓ) where
1313

14-
open import Algebra.Structures using (IsMagma)
15-
1614
open Monoid M
1715
using (Carrier; _∙_; _≈_; setoid; isMagma; semigroup; ε; sym; identityˡ
1816
; identityʳ ; ∙-cong; refl; assoc; ∙-congˡ; ∙-congʳ; trans)
@@ -51,7 +49,7 @@ open IntroElim public
5149

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

54-
cancelʳ : (b ∙ a) ∙ c ≈ b
52+
cancelʳ : (b ∙ a) ∙ c ≈ b
5553
cancelʳ = trans (assoc b a c) (trans (∙-congˡ inv) (identityʳ b))
5654

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

0 commit comments

Comments
 (0)