Skip to content

Commit 6bb39ce

Browse files
committed
refactor: use section-cong
1 parent 68e58cf commit 6bb39ce

File tree

1 file changed

+1
-2
lines changed

1 file changed

+1
-2
lines changed

src/Function/Properties/Bijection.agda

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -17,7 +17,6 @@ open import Relation.Binary.Definitions using (Reflexive; Trans)
1717
open import Relation.Binary.PropositionalEquality.Properties using (setoid)
1818
open import Data.Product.Base using (_,_; proj₁; proj₂)
1919
open import Function.Base using (_∘_)
20-
open import Function.Properties.Surjection using (injective⇒section-cong)
2120
open import Function.Properties.Inverse
2221
using (Inverse⇒Bijection; Inverse⇒Equivalence)
2322

@@ -39,7 +38,7 @@ Bijection⇒Inverse bij = record
3938
{ to = to
4039
; from = section
4140
; to-cong = cong
42-
; from-cong = injective⇒section-cong surjection injective
41+
; from-cong = Symmetry.section-cong bijective Eq₁.refl Eq₂.sym Eq₂.trans
4342
; inverse = section-inverseˡ
4443
, λ y≈to[x] injective (Eq₂.trans (section-strictInverseˡ _) y≈to[x])
4544
}

0 commit comments

Comments
 (0)