File tree Expand file tree Collapse file tree 1 file changed +4
-0
lines changed
Cubical/HITs/SetQuotients Expand file tree Collapse file tree 1 file changed +4
-0
lines changed Original file line number Diff line number Diff line change @@ -380,6 +380,10 @@ retract/R→section/R : {A : Type ℓ} {B : Type ℓ'} {R : A → A → Type ℓ
380380 section/R {iso/r = iso/r}
381381retract/R→section/R {R = R} {equivRel reflexive symmetric transitive} {iso/r = iso/r} b = iso/r .leftInv/R (iso/r .inv/R b)
382382
383+ -- Iso/R is a RelIso
384+ Iso/R→RelIso : {A : Type ℓ} {A' : Type ℓ'} {R : A → A → Type ℓ}{ER : isEquivRel R} → (iso/r : Iso/R A A' {R} ER) → RelIso {A = A} R {A' = A'} (R* {iso/r = iso/r})
385+ Iso/R→RelIso (iso/R fun/R₁ inv/R₁ leftInv/R₁) = reliso fun/R₁ inv/R₁ (λ a' → leftInv/R₁ (inv/R₁ a')) leftInv/R₁
386+
383387-- A 'natural' isomorphism/R when A ≡ B:
384388iso/R-A≡B : {A : Type ℓ} {B : Type ℓ} {R : A → A → Type ℓ}{ER : isEquivRel R} → (AB : A ≡ B) → Iso/R A B ER
385389iso/R-A≡B {ℓ} {A}{B}{R} ER@{equivRel reflexive symmetric transitive} AB .fun/R = λ z → transport AB z
You can’t perform that action at this time.
0 commit comments