Skip to content

Commit 0ecd8e0

Browse files
committed
Use _,_ rather than record syntax
1 parent bf1acf9 commit 0ecd8e0

File tree

1 file changed

+3
-8
lines changed

1 file changed

+3
-8
lines changed

src/Algebra/Construct/Quotient/Group.agda

Lines changed: 3 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -19,6 +19,7 @@ open import Algebra.Properties.Monoid monoid
1919
open import Algebra.Properties.Group G using (⁻¹-anti-homo-∙)
2020
open import Algebra.Structures using (IsGroup)
2121
open import Data.Product.Base using (_,_)
22+
open import Function.Base using (_∘_)
2223
open import Function.Definitions using (Surjective)
2324
open import Level using (_⊔_)
2425
open 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

0 commit comments

Comments
 (0)