Skip to content

Commit 6d725fd

Browse files
committed
refactor: use module ; rectify exported names
1 parent 2bcad3b commit 6d725fd

File tree

1 file changed

+6
-7
lines changed

1 file changed

+6
-7
lines changed

src/Function/Structures.agda

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

6868
open IsCongruent isCongruent public
6969

70-
private module IS = IsSurjective {≈₂ = _≈₂_} surjective
70+
private module S = Section _≈₂_ surjective
7171

72-
open IS public
73-
using (section; section-inverseˡ)
72+
open S public using (section; inverseˡ)
7473

7574
strictlySurjective : StrictlySurjective _≈₂_ f
76-
strictlySurjective = IS.strictlySurjective Eq₁.refl
75+
strictlySurjective = S.strictlySurjective Eq₁.refl
7776

78-
section-strictInverseˡ : StrictlyInverseˡ _≈₂_ f section
79-
section-strictInverseˡ _ = IS.section-inverseˡ Eq₁.refl
77+
strictlyInverseˡ : StrictlyInverseˡ _≈₂_ f section
78+
strictlyInverseˡ _ = S.inverseˡ Eq₁.refl
8079

8180

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

9897
open IsSurjection isSurjection public
99-
using (strictlySurjective; section; section-strictInverseˡ)
98+
using (strictlySurjective; section; inverseˡ; strictlyInverseˡ)
10099

101100

102101
------------------------------------------------------------------------

0 commit comments

Comments
 (0)