File tree Expand file tree Collapse file tree 3 files changed +7
-7
lines changed Expand file tree Collapse file tree 3 files changed +7
-7
lines changed Original file line number Diff line number Diff line change @@ -123,7 +123,7 @@ Additions to existing modules
123
123
inverseˡ : Inverseˡ _≈₁_ _≈₂_ to section
124
124
strictlyInverseˡ : StrictlyInverseˡ _≈₂_ to section
125
125
inverseʳ : Inverseʳ _≈₁_ _≈₂_ to section
126
- strictlyInverseʳ : StrictlyInverseʳ _≈₂_ section to
126
+ strictlyInverseʳ : StrictlyInverseʳ _≈₁_ to section
127
127
```
128
128
129
129
* In ` Function.Bundles.LeftInverse ` :
@@ -162,7 +162,7 @@ Additions to existing modules
162
162
inverseˡ : Inverseˡ _≈₁_ _≈₂_ f section
163
163
strictlyInverseˡ : StrictlyInverseˡ _≈₂_ f section
164
164
inverseʳ : Inverseʳ _≈₁_ _≈₂_ f section
165
- strictlyInverseʳ : StrictlyInverseʳ _≈₂_ section f
165
+ strictlyInverseʳ : StrictlyInverseʳ _≈₁_ f section
166
166
```
167
167
168
168
* In ` Function.Structures.IsSurjection ` :
Original file line number Diff line number Diff line change @@ -131,9 +131,6 @@ module Section (≈₂ : Rel B ℓ₂) (surj : Surjective {A = A} ≈₁ ≈₂
131
131
strictlyInverseˡ : StrictlyInverseˡ ≈₂ f section
132
132
strictlyInverseˡ _ = inverseˡ refl
133
133
134
- strictlyInverseʳ : StrictlyInverseʳ ≈₂ section f
135
- strictlyInverseʳ = strictlyInverseˡ
136
-
137
134
injective : Symmetric ≈₂ → Transitive ≈₂ → Injective ≈₂ ≈₁ section
138
135
injective sym trans = trans (sym (strictlyInverseˡ _)) ∘ inverseˡ
139
136
@@ -147,6 +144,9 @@ module Section (≈₂ : Rel B ℓ₂) (surj : Surjective {A = A} ≈₁ ≈₂
147
144
inverseʳ : Transitive ≈₂ → Inverseʳ ≈₁ ≈₂ f section
148
145
inverseʳ trans = inj ∘ trans (f∘section≡id _)
149
146
147
+ strictlyInverseʳ : Reflexive ≈₂ → Transitive ≈₂ → StrictlyInverseʳ ≈₁ f section
148
+ strictlyInverseʳ refl trans _ = inverseʳ trans refl
149
+
150
150
surjective : Transitive ≈₂ → Surjective ≈₂ ≈₁ section
151
151
surjective trans x = f x , inverseʳ trans
152
152
Original file line number Diff line number Diff line change @@ -102,8 +102,8 @@ record IsBijection (f : A → B) : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
102
102
inverseʳ : Inverseʳ _≈₁_ _≈₂_ f section
103
103
inverseʳ = S.inverseʳ injective Eq₁.refl Eq₂.trans
104
104
105
- strictlyInverseʳ : StrictlyInverseʳ _≈₂_ section f
106
- strictlyInverseʳ = S.strictlyInverseʳ Eq₁ .refl
105
+ strictlyInverseʳ : StrictlyInverseʳ _≈₁_ f section
106
+ strictlyInverseʳ _ = inverseʳ Eq₂ .refl
107
107
108
108
109
109
------------------------------------------------------------------------
You can’t perform that action at this time.
0 commit comments