File tree Expand file tree Collapse file tree 1 file changed +3
-2
lines changed
src/Algebra/Construct/Centre Expand file tree Collapse file tree 1 file changed +3
-2
lines changed Original file line number Diff line number Diff line change @@ -13,11 +13,12 @@ module Algebra.Construct.Centre.Monoid
1313 {c ℓ} (monoid : Monoid c ℓ)
1414 where
1515
16- open import Algebra.Consequences.Setoid using (identity⇒central)
1716open import Algebra.Morphism.Structures
1817open import Algebra.Morphism.MonoidMonomorphism using (isMonoid)
1918open import Function.Base using (id)
2019
20+ open import Algebra.Properties.Monoid monoid using (ε-central)
21+
2122private
2223 module G = Monoid monoid
2324
@@ -35,7 +36,7 @@ open import Algebra.Construct.Centre.Semigroup G.semigroup as Z public
3536ε : Center
3637ε = record
3738 { ι = G.ε
38- ; central = identity⇒ central G.setoid {_∙_ = G._∙_} G.identity
39+ ; central = ε- central
3940 }
4041
4142domain : RawMonoid _ _
You can’t perform that action at this time.
0 commit comments