File tree Expand file tree Collapse file tree 1 file changed +3
-8
lines changed
src/Algebra/Construct/Quotient Expand file tree Collapse file tree 1 file changed +3
-8
lines changed Original file line number Diff line number Diff line change @@ -19,6 +19,7 @@ open import Algebra.Properties.Monoid monoid
1919open import Algebra.Properties.Group G using (⁻¹-anti-homo-∙)
2020open import Algebra.Structures using (IsGroup)
2121open import Data.Product.Base using (_,_)
22+ open import Function.Base using (_∘_)
2223open import Function.Definitions using (Surjective)
2324open import Level using (_⊔_)
2425open import Relation.Binary.Core using (_⇒_)
@@ -90,15 +91,9 @@ quotientIsGroup = record
9091 }
9192 ; assoc = λ x y z → ≈⇒≋ (assoc x y z)
9293 }
93- ; identity = record
94- { fst = λ x → ≈⇒≋ (identityˡ x)
95- ; snd = λ x → ≈⇒≋ (identityʳ x)
96- }
97- }
98- ; inverse = record
99- { fst = λ x → ≈⇒≋ (inverseˡ x)
100- ; snd = λ x → ≈⇒≋ (inverseʳ x)
94+ ; identity = ≈⇒≋ ∘ identityˡ , ≈⇒≋ ∘ identityʳ
10195 }
96+ ; inverse = ≈⇒≋ ∘ inverseˡ , ≈⇒≋ ∘ inverseʳ
10297 ; ⁻¹-cong = ≋-⁻¹-cong
10398 }
10499
You can’t perform that action at this time.
0 commit comments