Skip to content

Commit

Permalink
refactor: use section-cong
Browse files Browse the repository at this point in the history
  • Loading branch information
jamesmckinna committed Jan 30, 2025
1 parent 68e58cf commit 6bb39ce
Showing 1 changed file with 1 addition and 2 deletions.
3 changes: 1 addition & 2 deletions src/Function/Properties/Bijection.agda
Original file line number Diff line number Diff line change
Expand Up @@ -17,7 +17,6 @@ open import Relation.Binary.Definitions using (Reflexive; Trans)
open import Relation.Binary.PropositionalEquality.Properties using (setoid)
open import Data.Product.Base using (_,_; proj₁; proj₂)
open import Function.Base using (_∘_)
open import Function.Properties.Surjection using (injective⇒section-cong)
open import Function.Properties.Inverse
using (Inverse⇒Bijection; Inverse⇒Equivalence)

Expand All @@ -39,7 +38,7 @@ Bijection⇒Inverse bij = record
{ to = to
; from = section
; to-cong = cong
; from-cong = injective⇒section-cong surjection injective
; from-cong = Symmetry.section-cong bijective Eq₁.refl Eq₂.sym Eq₂.trans
; inverse = section-inverseˡ
, λ y≈to[x] injective (Eq₂.trans (section-strictInverseˡ _) y≈to[x])
}
Expand Down

0 comments on commit 6bb39ce

Please sign in to comment.