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