File tree Expand file tree Collapse file tree 1 file changed +2
-2
lines changed Expand file tree Collapse file tree 1 file changed +2
-2
lines changed Original file line number Diff line number Diff line change @@ -60,7 +60,7 @@ record IsInjection (to : A → B) : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
60
60
open IsCongruent isCongruent public
61
61
62
62
63
- record IsSurjection (f : A → B) : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
63
+ record IsSurjection (f : A → B ) : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
64
64
field
65
65
isCongruent : IsCongruent f
66
66
surjective : Surjective _≈₁_ _≈₂_ f
@@ -103,7 +103,7 @@ record IsBijection (f : A → B) : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
103
103
inverseʳ = S.inverseʳ injective Eq₁.refl Eq₂.trans
104
104
105
105
strictlyInverseʳ : StrictlyInverseʳ _≈₂_ section f
106
- strictlyInverseʳ = S.strictlyInverseʳ injective Eq₁.refl Eq₂.trans
106
+ strictlyInverseʳ = S.strictlyInverseʳ Eq₁.refl
107
107
108
108
109
109
------------------------------------------------------------------------
You can’t perform that action at this time.
0 commit comments