Skip to content

Commit 53ab09a

Browse files
committed
refactor: propagate exports of new lemmas
1 parent 1439887 commit 53ab09a

File tree

2 files changed

+10
-1
lines changed

2 files changed

+10
-1
lines changed

src/Function/Bundles.agda

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -172,7 +172,8 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
172172
; surjective = surjective
173173
}
174174

175-
open IsBijection isBijection public using (module Eq₁; module Eq₂)
175+
open IsBijection isBijection public
176+
using (module Eq₁; module Eq₂; inverseʳ; strictlyInverseʳ)
176177

177178

178179
------------------------------------------------------------------------

src/Function/Structures.agda

Lines changed: 8 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -97,6 +97,14 @@ record IsBijection (f : A → B) : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
9797
open IsSurjection isSurjection public
9898
using (strictlySurjective; section; inverseˡ; strictlyInverseˡ)
9999

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+
100108

101109
------------------------------------------------------------------------
102110
-- Two element structures

0 commit comments

Comments
 (0)