Skip to content

Commit a4f3cb2

Browse files
committed
Promote some isomorphisms of truncations to equivalences
1 parent fdaa6cf commit a4f3cb2

File tree

1 file changed

+7
-0
lines changed

1 file changed

+7
-0
lines changed

Cubical/HITs/Truncation/Properties.agda

Lines changed: 7 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -316,6 +316,9 @@ Iso.inv (mapCompIso {n = (suc n)} g) = map (Iso.inv g)
316316
Iso.rightInv (mapCompIso {n = (suc n)} g) = elim (λ x isOfHLevelPath _ (isOfHLevelTrunc _) _ _) λ b cong ∣_∣ (Iso.rightInv g b)
317317
Iso.leftInv (mapCompIso {n = (suc n)} g) = elim (λ x isOfHLevelPath _ (isOfHLevelTrunc _) _ _) λ a cong ∣_∣ (Iso.leftInv g a)
318318

319+
mapCompEquiv : {n : HLevel} {B : Type ℓ'} (A ≃ B) (hLevelTrunc n A) ≃ (hLevelTrunc n B)
320+
mapCompEquiv e = isoToEquiv (mapCompIso (equivToIso e))
321+
319322
mapId : {n : HLevel} t map {n = n} (idfun A) t ≡ t
320323
mapId {n = 0} tt* = refl
321324
mapId {n = (suc n)} =
@@ -576,6 +579,10 @@ Iso.rightInv (truncOfΣIso (suc n)) =
576579
Iso.leftInv (truncOfΣIso (suc n)) =
577580
elim (λ _ isOfHLevelPath (suc n) (isOfHLevelTrunc (suc n)) _ _) λ {(a , b) refl}
578581

582+
truncOfΣEquiv : {ℓ ℓ'} (n : HLevel) {A : Type ℓ} {B : A Type ℓ'}
583+
(hLevelTrunc n (Σ A B)) ≃ (hLevelTrunc n (Σ A (hLevelTrunc n ∘ B)))
584+
truncOfΣEquiv n = isoToEquiv (truncOfΣIso n)
585+
579586
{- transport along family of truncations -}
580587

581588
transportTrunc : {n : HLevel}{p : A ≡ B}

0 commit comments

Comments
 (0)