File tree Expand file tree Collapse file tree 2 files changed +10
-1
lines changed Expand file tree Collapse file tree 2 files changed +10
-1
lines changed Original file line number Diff line number Diff line change @@ -172,7 +172,8 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
172
172
; surjective = surjective
173
173
}
174
174
175
- open IsBijection isBijection public using (module Eq₁ ; module Eq₂ )
175
+ open IsBijection isBijection public
176
+ using (module Eq₁ ; module Eq₂ ; inverseʳ; strictlyInverseʳ)
176
177
177
178
178
179
------------------------------------------------------------------------
Original file line number Diff line number Diff line change @@ -97,6 +97,14 @@ record IsBijection (f : A → B) : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
97
97
open IsSurjection isSurjection public
98
98
using (strictlySurjective; section; inverseˡ; strictlyInverseˡ)
99
99
100
+ private module S = Section _≈₂_ surjective
101
+
102
+ inverseʳ : Inverseʳ _≈₁_ _≈₂_ f section
103
+ inverseʳ = S.inverseʳ injective Eq₁.refl Eq₂.trans
104
+
105
+ strictlyInverseʳ : StrictlyInverseʳ _≈₂_ section f
106
+ strictlyInverseʳ = S.strictlyInverseʳ injective Eq₁.refl Eq₂.trans
107
+
100
108
101
109
------------------------------------------------------------------------
102
110
-- Two element structures
You can’t perform that action at this time.
0 commit comments