Skip to content

Commit

Permalink
Remove an unnecessary argument in aurefl (#801)
Browse files Browse the repository at this point in the history
  • Loading branch information
vikraman committed May 17, 2022
1 parent b6fbca9 commit c24289d
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions Cubical/Foundations/Univalence.agda
Original file line number Diff line number Diff line change
Expand Up @@ -172,15 +172,15 @@ EquivJ P r e = subst (λ x → P (x .fst) (x .snd)) (contrSinglEquiv e) r

-- Assuming that we have an inverse to ua we can easily prove univalence
module Univalence (au : {ℓ} {A B : Type ℓ} A ≡ B A ≃ B)
(aurefl : {ℓ} {A B : Type ℓ} au refl ≡ idEquiv A) where
(aurefl : {ℓ} {A : Type ℓ} au refl ≡ idEquiv A) where

ua-au : {A B : Type ℓ} (p : A ≡ B) ua (au p) ≡ p
ua-au {B = B} = J (λ _ p ua (au p) ≡ p)
(cong ua (aurefl {B = B}) ∙ uaIdEquiv)
(cong ua aurefl ∙ uaIdEquiv)

au-ua : {A B : Type ℓ} (e : A ≃ B) au (ua e) ≡ e
au-ua {B = B} = EquivJ (λ _ f au (ua f) ≡ f)
(subst (λ r au r ≡ idEquiv _) (sym uaIdEquiv) (aurefl {B = B}))
(subst (λ r au r ≡ idEquiv _) (sym uaIdEquiv) aurefl)

isoThm : {ℓ} {A B : Type ℓ} Iso (A ≡ B) (A ≃ B)
isoThm .Iso.fun = au
Expand Down

0 comments on commit c24289d

Please sign in to comment.