Skip to content

Commit e6899ef

Browse files
committed
refactor: re-export from Consequences.IsSurjective
1 parent 2f6b3c2 commit e6899ef

File tree

1 file changed

+7
-8
lines changed

1 file changed

+7
-8
lines changed

src/Function/Structures.agda

Lines changed: 7 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -67,17 +67,16 @@ record IsSurjection (f : A → B) : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
6767

6868
open IsCongruent isCongruent public
6969

70-
strictlySurjective : StrictlySurjective _≈₂_ f
71-
strictlySurjective = surjective⇒strictlySurjective _≈₂_ Eq₁.refl surjective
70+
private module IS = IsSurjective {≈₂ = _≈₂_} surjective
7271

73-
section : B A
74-
section = proj₁ ∘ surjective
72+
open IS public
73+
using (section; section-inverseˡ)
7574

76-
section-inverseˡ : Inverseˡ _≈₁_ _≈₂_ f section
77-
section-inverseˡ {x = x} = proj₂ (surjective x)
75+
strictlySurjective : StrictlySurjective _≈₂_ f
76+
strictlySurjective = IS.strictlySurjective Eq₁.refl
7877

7978
section-strictInverseˡ : StrictlyInverseˡ _≈₂_ f section
80-
section-strictInverseˡ _ = section-inverseˡ Eq₁.refl
79+
section-strictInverseˡ _ = IS.section-inverseˡ Eq₁.refl
8180

8281

8382
record IsBijection (f : A B) : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
@@ -97,7 +96,7 @@ record IsBijection (f : A → B) : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
9796
}
9897

9998
open IsSurjection isSurjection public
100-
using (strictlySurjective; section)
99+
using (strictlySurjective; section; section-strictInverseˡ)
101100

102101

103102
------------------------------------------------------------------------

0 commit comments

Comments
 (0)