Skip to content

Commit

Permalink
Add 2 argument version of ua→ (#713)
Browse files Browse the repository at this point in the history
  • Loading branch information
shlevy committed Feb 3, 2022
1 parent 9acdecf commit ccf7c01
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions Cubical/Foundations/Univalence.agda
Original file line number Diff line number Diff line change
Expand Up @@ -263,6 +263,14 @@ ua→⁻ {e = e} {f₀ = f₀} {f₁} p a i =
})
(p i (transp (λ j ua e (j ∧ i)) (~ i) a))

ua→2 : {ℓ ℓ' ℓ''} {A₀ A₁ : Type ℓ} {e₁ : A₀ ≃ A₁}
{B₀ B₁ : Type ℓ'} {e₂ : B₀ ≃ B₁}
{C : (i : I) Type ℓ''}
{f₀ : A₀ B₀ C i0} {f₁ : A₁ B₁ C i1}
( a b PathP C (f₀ a b) (f₁ (e₁ .fst a) (e₂ .fst b)))
PathP (λ i ua e₁ i ua e₂ i C i) f₀ f₁
ua→2 h = ua→ (ua→ ∘ h)

-- Useful lemma for unfolding a transported function over ua
-- If we would have regularity this would be refl
transportUAop₁ : {A B : Type ℓ} (e : A ≃ B) (f : A A) (x : B)
Expand Down

0 comments on commit ccf7c01

Please sign in to comment.