File tree Expand file tree Collapse file tree 1 file changed +8
-2
lines changed Expand file tree Collapse file tree 1 file changed +8
-2
lines changed Original file line number Diff line number Diff line change 1+ ------------------------------------------------------------------------
2+ -- The Agda standard library
3+ --
4+ -- Equational reasoning for monoids
5+ -- (Utilities for identity and cancellation reasoning, extending semigroup reasoning)
6+ ------------------------------------------------------------------------
7+
18{-# OPTIONS --cubical-compatible --safe #-}
29
310open import Algebra using (Monoid)
@@ -6,8 +13,7 @@ module Algebra.Reasoning.Monoid {o ℓ} (M : Monoid o ℓ) where
613
714open Monoid M
815open import Relation.Binary.Reasoning.Setoid setoid
9- open import Algebra.Reasoning.SemiGroup semigroup public
10-
16+ open import Algebra.Reasoning.Semigroup semigroup public
1117
1218module Identity {a : Carrier } where
1319 id-unique : (∀ b → b ∙ a ≈ b) → a ≈ ε
You can’t perform that action at this time.
0 commit comments