-
Notifications
You must be signed in to change notification settings - Fork 256
Closed
Description
Obviously Maybe a case of mis-subclassing. It leads to unobvious requirements and also makes the record much longer than it needs to be.
agda-stdlib/src/Algebra/Structures.agda
Lines 45 to 51 in a0bdb8e
record IsCommutativeMonoid {a ℓ} {A : Set a} (≈ : Rel A ℓ) | |
(_∙_ : Op₂ A) (ε : A) : Set (a ⊔ ℓ) where | |
open FunctionProperties ≈ | |
field | |
isSemigroup : IsSemigroup ≈ _∙_ | |
identityˡ : LeftIdentity ε _∙_ | |
comm : Commutative _∙_ |