Skip to content

Commit ff966fe

Browse files
committed
Syntax modification
1 parent 41696ed commit ff966fe

File tree

1 file changed

+8
-2
lines changed

1 file changed

+8
-2
lines changed

src/Algebra/Reasoning/Monoid.agda

Lines changed: 8 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,10 @@
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

310
open import Algebra using (Monoid)
@@ -6,8 +13,7 @@ module Algebra.Reasoning.Monoid {o ℓ} (M : Monoid o ℓ) where
613

714
open Monoid M
815
open import Relation.Binary.Reasoning.Setoid setoid
9-
open import Algebra.Reasoning.SemiGroup semigroup public
10-
16+
open import Algebra.Reasoning.Semigroup semigroup public
1117

1218
module Identity {a : Carrier } where
1319
id-unique : ( b b ∙ a ≈ b) a ≈ ε

0 commit comments

Comments
 (0)