File tree Expand file tree Collapse file tree 1 file changed +6
-7
lines changed Expand file tree Collapse file tree 1 file changed +6
-7
lines changed Original file line number Diff line number Diff line change @@ -67,16 +67,15 @@ record IsSurjection (f : A → B) : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
67
67
68
68
open IsCongruent isCongruent public
69
69
70
- private module IS = IsSurjective {≈₂ = _≈₂_} surjective
70
+ private module S = Section _≈₂_ surjective
71
71
72
- open IS public
73
- using (section; section-inverseˡ)
72
+ open S public using (section; inverseˡ)
74
73
75
74
strictlySurjective : StrictlySurjective _≈₂_ f
76
- strictlySurjective = IS .strictlySurjective Eq₁.refl
75
+ strictlySurjective = S .strictlySurjective Eq₁.refl
77
76
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
80
79
81
80
82
81
record IsBijection (f : A → B) : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
@@ -96,7 +95,7 @@ record IsBijection (f : A → B) : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
96
95
}
97
96
98
97
open IsSurjection isSurjection public
99
- using (strictlySurjective; section; section-strictInverseˡ )
98
+ using (strictlySurjective; section; inverseˡ; strictlyInverseˡ )
100
99
101
100
102
101
------------------------------------------------------------------------
You can’t perform that action at this time.
0 commit comments