Properties of equivalences depending on function extensionality.

(Not included in UF-Equiv because the module funext defines function
extensionality as the equivalence of happly for suitable parameters.)

\begin{code}

{-# OPTIONS --without-K --exact-split --safe #-}

module UF-Equiv-FunExt where

open import SpartanMLTT
open import UF-Base
open import UF-Subsingletons
open import UF-Subsingletons-FunExt
open import UF-Retracts
open import UF-FunExt
open import UF-Equiv
open import UF-EquivalenceExamples

being-vv-equiv-is-prop' : funext ๐“ฅ (๐“ค โŠ” ๐“ฅ) โ†’ funext (๐“ค โŠ” ๐“ฅ) (๐“ค โŠ” ๐“ฅ)
                        โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } (f : X โ†’ Y)
                        โ†’ is-prop (is-vv-equiv f)
being-vv-equiv-is-prop' {๐“ค} {๐“ฅ} fe fe' f = ฮ -is-prop
                                             fe
                                             (ฮป x โ†’ being-singleton-is-prop fe' )

being-vv-equiv-is-prop : FunExt
                       โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } (f : X โ†’ Y)
                       โ†’ is-prop (is-vv-equiv f)
being-vv-equiv-is-prop {๐“ค} {๐“ฅ} fe = being-vv-equiv-is-prop' (fe ๐“ฅ (๐“ค โŠ” ๐“ฅ)) (fe (๐“ค โŠ” ๐“ฅ) (๐“ค โŠ” ๐“ฅ))

qinv-post' : {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } {A : ๐“ฆ ฬ‡ }
          โ†’ naive-funext ๐“ฆ ๐“ค โ†’ naive-funext ๐“ฆ ๐“ฅ
          โ†’ (f : X โ†’ Y) โ†’ qinv f โ†’ qinv (ฮป (h : A โ†’ X) โ†’ f โˆ˜ h)
qinv-post' {๐“ค} {๐“ฅ} {๐“ฆ} {X} {Y} {A} nfe nfe' f (g , ฮท , ฮต) = (g' , ฮท' , ฮต')
 where
  f' : (A โ†’ X) โ†’ (A โ†’ Y)
  f' h = f โˆ˜ h
  g' : (A โ†’ Y) โ†’ (A โ†’ X)
  g' k = g โˆ˜ k
  ฮท' : (h : A โ†’ X) โ†’ g' (f' h) โ‰ก h
  ฮท' h = nfe (ฮท โˆ˜ h)
  ฮต' : (k : A โ†’ Y) โ†’ f' (g' k) โ‰ก k
  ฮต' k = nfe' (ฮต โˆ˜ k)

qinv-post : (โˆ€ ๐“ค ๐“ฅ โ†’ naive-funext ๐“ค ๐“ฅ) โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } {A : ๐“ฆ ฬ‡ } (f : X โ†’ Y)
          โ†’ qinv f โ†’ qinv (ฮป (h : A โ†’ X) โ†’ f โˆ˜ h)
qinv-post {๐“ค} {๐“ฅ} {๐“ฆ} nfe = qinv-post' (nfe ๐“ฆ ๐“ค) (nfe ๐“ฆ ๐“ฅ)

equiv-post : {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } {A : ๐“ฆ ฬ‡ }
           โ†’ naive-funext ๐“ฆ ๐“ค โ†’ naive-funext ๐“ฆ ๐“ฅ
           โ†’ (f : X โ†’ Y) โ†’ is-equiv f โ†’ is-equiv (ฮป (h : A โ†’ X) โ†’ f โˆ˜ h)
equiv-post nfe nfe' f e = qinvs-are-equivs (ฮป h โ†’ f โˆ˜ h) (qinv-post' nfe nfe' f (equivs-are-qinvs f e))

qinv-pre' : {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } {A : ๐“ฆ ฬ‡ }
          โ†’ naive-funext ๐“ฅ ๐“ฆ โ†’ naive-funext ๐“ค ๐“ฆ
          โ†’ (f : X โ†’ Y) โ†’ qinv f โ†’ qinv (ฮป (h : Y โ†’ A) โ†’ h โˆ˜ f)
qinv-pre' {๐“ค} {๐“ฅ} {๐“ฆ} {X} {Y} {A} nfe nfe' f (g , ฮท , ฮต) = (g' , ฮท' , ฮต')
 where
  f' : (Y โ†’ A) โ†’ (X โ†’ A)
  f' h = h โˆ˜ f
  g' : (X โ†’ A) โ†’ (Y โ†’ A)
  g' k = k โˆ˜ g
  ฮท' : (h : Y โ†’ A) โ†’ g' (f' h) โ‰ก h
  ฮท' h = nfe (ฮป y โ†’ ap h (ฮต y))
  ฮต' : (k : X โ†’ A) โ†’ f' (g' k) โ‰ก k
  ฮต' k = nfe' (ฮป x โ†’ ap k (ฮท x))

qinv-pre : (โˆ€ ๐“ค ๐“ฅ โ†’ naive-funext ๐“ค ๐“ฅ) โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } {A : ๐“ฆ ฬ‡ } (f : X โ†’ Y)
         โ†’ qinv f โ†’ qinv (ฮป (h : Y โ†’ A) โ†’ h โˆ˜ f)
qinv-pre {๐“ค} {๐“ฅ} {๐“ฆ} nfe = qinv-pre' (nfe ๐“ฅ ๐“ฆ) (nfe ๐“ค ๐“ฆ)

retractions-have-at-most-one-section' : {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ }
                                      โ†’ funext ๐“ฅ ๐“ค โ†’ funext ๐“ฅ ๐“ฅ
                                      โ†’ (f : X โ†’ Y) โ†’ is-section f โ†’ is-prop (has-section f)
retractions-have-at-most-one-section' {๐“ค} {๐“ฅ} {X} {Y} fe fe' f (g , gf) (h , fh) =
 singletons-are-props c (h , fh)
 where
  a : qinv f
  a = equivs-are-qinvs f ((h , fh) , g , gf)
  b : is-singleton(fiber (ฮป h โ†’  f โˆ˜ h) id)
  b = qinvs-are-vv-equivs (ฮป h โ†’  f โˆ˜ h) (qinv-post' (dfunext fe) (dfunext fe') f a) id
  r : fiber (ฮป h โ†’  f โˆ˜ h) id โ†’ has-section f
  r (h , p) = (h , happly' (f โˆ˜ h) id p)
  s : has-section f โ†’ fiber (ฮป h โ†’  f โˆ˜ h) id
  s (h , ฮท) = (h , dfunext fe' ฮท)
  rs : (ฯƒ : has-section f) โ†’ r (s ฯƒ) โ‰ก ฯƒ
  rs (h , ฮท) = ap (ฮป - โ†’ (h , -)) q
   where
    q : happly' (f โˆ˜ h) id (dfunext fe' ฮท) โ‰ก ฮท
    q = happly-funext fe' (f โˆ˜ h) id ฮท
  c : is-singleton (has-section f)
  c = retract-of-singleton (r , s , rs) b

sections-have-at-most-one-retraction' : {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ }
                                      โ†’ funext ๐“ค ๐“ค โ†’ funext ๐“ฅ ๐“ค
                                      โ†’ (f : X โ†’ Y) โ†’ has-section f โ†’ is-prop (is-section f)
sections-have-at-most-one-retraction' {๐“ค} {๐“ฅ} {X} {Y} fe fe' f (g , fg) (h , hf) =
 singletons-are-props c (h , hf)
 where
  a : qinv f
  a = equivs-are-qinvs f ((g , fg) , (h , hf))
  b : is-singleton(fiber (ฮป h โ†’  h โˆ˜ f) id)
  b = qinvs-are-vv-equivs (ฮป h โ†’  h โˆ˜ f) (qinv-pre' (dfunext fe') (dfunext fe) f a) id
  r : fiber (ฮป h โ†’  h โˆ˜ f) id โ†’ is-section f
  r (h , p) = (h , happly' (h โˆ˜ f) id p)
  s : is-section f โ†’ fiber (ฮป h โ†’  h โˆ˜ f) id
  s (h , ฮท) = (h , dfunext fe ฮท)
  rs : (ฯƒ : is-section f) โ†’ r (s ฯƒ) โ‰ก ฯƒ
  rs (h , ฮท) = ap (ฮป - โ†’ (h , -)) q
   where
    q : happly' (h โˆ˜ f) id (dfunext fe ฮท) โ‰ก ฮท
    q = happly-funext fe (h โˆ˜ f) id ฮท
  c : is-singleton (is-section f)
  c = retract-of-singleton (r , s , rs) b

retractions-have-at-most-one-section : FunExt โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } (f : X โ†’ Y)
                                     โ†’ is-section f โ†’ is-prop (has-section f)
retractions-have-at-most-one-section {๐“ค} {๐“ฅ} fe = retractions-have-at-most-one-section' (fe ๐“ฅ ๐“ค) (fe ๐“ฅ ๐“ฅ)

sections-have-at-most-one-retraction : FunExt โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } (f : X โ†’ Y)
                                     โ†’ has-section f โ†’ is-prop (is-section f)
sections-have-at-most-one-retraction {๐“ค} {๐“ฅ} fe = sections-have-at-most-one-retraction' (fe ๐“ค ๐“ค) (fe ๐“ฅ ๐“ค)

being-equiv-is-prop' : {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ }
                     โ†’ funext ๐“ฅ ๐“ค โ†’ funext ๐“ฅ ๐“ฅ โ†’ funext ๐“ค ๐“ค โ†’ funext ๐“ฅ ๐“ค
                     โ†’ (f : X โ†’ Y) โ†’ is-prop (is-equiv f)
being-equiv-is-prop' fe fe' fe'' fe''' f = ร—-prop-criterion (retractions-have-at-most-one-section' fe fe' f ,
                                                               sections-have-at-most-one-retraction' fe'' fe''' f)

being-equiv-is-prop : FunExt โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } (f : X โ†’ Y)
                    โ†’ is-prop (is-equiv f)
being-equiv-is-prop {๐“ค} {๐“ฅ} fe f = being-equiv-is-prop' (fe ๐“ฅ ๐“ค) (fe ๐“ฅ ๐“ฅ) (fe ๐“ค ๐“ค) (fe ๐“ฅ ๐“ค) f

being-equiv-is-prop'' : {X Y : ๐“ค ฬ‡ }
                      โ†’ funext ๐“ค ๐“ค
                      โ†’ (f : X โ†’ Y) โ†’ is-prop (is-equiv f)
being-equiv-is-prop'' fe = being-equiv-is-prop' fe fe fe fe

โ‰ƒ-assoc : FunExt
        โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } {Z : ๐“ฆ ฬ‡ } {T : ๐“ฃ ฬ‡ }
          (ฮฑ : X โ‰ƒ Y) (ฮฒ : Y โ‰ƒ Z) (ฮณ : Z โ‰ƒ T)
        โ†’ ฮฑ โ— (ฮฒ โ— ฮณ) โ‰ก (ฮฑ โ— ฮฒ) โ— ฮณ
โ‰ƒ-assoc fe (f , a) (g , b) (h , c) = to-ฮฃ-โ‰ก (p , q)
 where
  p : (h โˆ˜ g) โˆ˜ f โ‰ก h โˆ˜ (g โˆ˜ f)
  p = refl

  d e : is-equiv (h โˆ˜ g โˆ˜ f)
  d = โˆ˜-is-equiv a (โˆ˜-is-equiv b c)
  e = โˆ˜-is-equiv (โˆ˜-is-equiv a b) c

  q : transport is-equiv p d โ‰ก e
  q = being-equiv-is-prop fe (h โˆ˜ g โˆ˜ f) _ _

\end{code}

The above proof can be condensed to one line in the style of the
following two proofs, which exploit the fact that the identity map is
a neutral element for ordinary function composition, definitionally:

\begin{code}

โ‰ƒ-refl-left' : funext ๐“ฅ ๐“ค โ†’ funext ๐“ฅ ๐“ฅ โ†’ funext ๐“ค ๐“ค
               โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } (ฮฑ : X โ‰ƒ Y) โ†’ โ‰ƒ-refl X โ— ฮฑ โ‰ก ฮฑ
โ‰ƒ-refl-left' feโ‚€ feโ‚ feโ‚‚ ฮฑ = to-ฮฃ-โ‰ก' (being-equiv-is-prop' feโ‚€ feโ‚ feโ‚‚ feโ‚€ _ _ _)

โ‰ƒ-refl-right' : funext ๐“ฅ ๐“ค โ†’ funext ๐“ฅ ๐“ฅ โ†’ funext ๐“ค ๐“ค โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } (ฮฑ : X โ‰ƒ Y) โ†’ ฮฑ โ— โ‰ƒ-refl Y โ‰ก ฮฑ
โ‰ƒ-refl-right' feโ‚€ feโ‚ feโ‚‚  ฮฑ = to-ฮฃ-โ‰ก' (being-equiv-is-prop' feโ‚€ feโ‚ feโ‚‚ feโ‚€ _ _ _)

โ‰ƒ-sym-involutive' : funext ๐“ฅ ๐“ค โ†’ funext ๐“ฅ ๐“ฅ โ†’ funext ๐“ค ๐“ค
                  โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } (ฮฑ : X โ‰ƒ Y) โ†’ โ‰ƒ-sym (โ‰ƒ-sym ฮฑ) โ‰ก ฮฑ
โ‰ƒ-sym-involutive' feโ‚€ feโ‚ feโ‚‚ (f , a) = to-ฮฃ-โ‰ก
                                             (inversion-involutive f a ,
                                              being-equiv-is-prop' feโ‚€ feโ‚ feโ‚‚ feโ‚€ f _ a)

โ‰ƒ-Sym' : funext ๐“ฅ ๐“ค โ†’ funext ๐“ฅ ๐“ฅ โ†’ funext ๐“ค ๐“ค โ†’ funext ๐“ค ๐“ฅ
       โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } โ†’ (X โ‰ƒ Y) โ‰ƒ (Y โ‰ƒ X)
โ‰ƒ-Sym' feโ‚€ feโ‚ feโ‚‚ feโ‚ƒ = qinveq โ‰ƒ-sym (โ‰ƒ-sym , โ‰ƒ-sym-involutive' feโ‚€ feโ‚ feโ‚‚ , โ‰ƒ-sym-involutive' feโ‚ƒ feโ‚‚ feโ‚)

โ‰ƒ-Sym'' : funext ๐“ค ๐“ค
        โ†’ {X Y : ๐“ค ฬ‡ } โ†’ (X โ‰ƒ Y) โ‰ƒ (Y โ‰ƒ X)
โ‰ƒ-Sym'' fe = โ‰ƒ-Sym' fe fe fe fe

โ‰ƒ-Sym : FunExt โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } โ†’ (X โ‰ƒ Y) โ‰ƒ (Y โ‰ƒ X)
โ‰ƒ-Sym {๐“ค} {๐“ฅ} fe = โ‰ƒ-Sym' (fe ๐“ฅ ๐“ค) (fe ๐“ฅ ๐“ฅ) (fe ๐“ค ๐“ค) (fe ๐“ค ๐“ฅ)

โ‰ƒ-refl-left : FunExt โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } (ฮฑ : X โ‰ƒ Y) โ†’ โ‰ƒ-refl X โ— ฮฑ โ‰ก ฮฑ
โ‰ƒ-refl-left fe = โ‰ƒ-refl-left' (fe _ _) (fe _ _) (fe _ _)

โ‰ƒ-refl-right : FunExt โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } (ฮฑ : X โ‰ƒ Y) โ†’ ฮฑ โ— โ‰ƒ-refl Y โ‰ก ฮฑ
โ‰ƒ-refl-right fe = โ‰ƒ-refl-right' (fe _ _) (fe _ _) (fe _ _)

โ‰ƒ-sym-involutive : FunExt โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } (ฮฑ : X โ‰ƒ Y) โ†’ โ‰ƒ-sym (โ‰ƒ-sym ฮฑ) โ‰ก ฮฑ
โ‰ƒ-sym-involutive {๐“ค} {๐“ฅ} fe = โ‰ƒ-sym-involutive' (fe ๐“ฅ ๐“ค) (fe ๐“ฅ ๐“ฅ) (fe ๐“ค ๐“ค)

โ‰ƒ-sym-left-inverse : FunExt โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } (ฮฑ : X โ‰ƒ Y) โ†’ โ‰ƒ-sym ฮฑ โ— ฮฑ โ‰ก โ‰ƒ-refl Y
โ‰ƒ-sym-left-inverse {๐“ค} {๐“ฅ} fe (f , e) = to-ฮฃ-โ‰ก (p , being-equiv-is-prop fe _ _ _)
 where
  p : f โˆ˜ inverse f e โ‰ก id
  p = dfunext (fe ๐“ฅ ๐“ฅ) (inverses-are-sections f e)

โ‰ƒ-sym-right-inverse : FunExt โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } (ฮฑ : X โ‰ƒ Y) โ†’ ฮฑ โ— โ‰ƒ-sym ฮฑ โ‰ก โ‰ƒ-refl X
โ‰ƒ-sym-right-inverse {๐“ค} {๐“ฅ} fe (f , e) = to-ฮฃ-โ‰ก (p , being-equiv-is-prop fe _ _ _)
 where
  p : inverse f e โˆ˜ f โ‰ก id
  p = dfunext (fe ๐“ค ๐“ค) (inverses-are-retractions f e)

โ‰ƒ-Comp : FunExt โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } (Z : ๐“ฆ ฬ‡ ) โ†’ X โ‰ƒ Y โ†’ (Y โ‰ƒ Z) โ‰ƒ (X โ‰ƒ Z)
โ‰ƒ-Comp fe Z ฮฑ = qinveq (ฮฑ โ—_) ((โ‰ƒ-sym ฮฑ โ—_), p , q)
 where
  p = ฮป ฮฒ โ†’ โ‰ƒ-sym ฮฑ โ— (ฮฑ โ— ฮฒ) โ‰กโŸจ โ‰ƒ-assoc fe (โ‰ƒ-sym ฮฑ) ฮฑ ฮฒ โŸฉ
            (โ‰ƒ-sym ฮฑ โ— ฮฑ) โ— ฮฒ โ‰กโŸจ ap (_โ— ฮฒ) (โ‰ƒ-sym-left-inverse fe ฮฑ) โŸฉ
            โ‰ƒ-refl _ โ— ฮฒ      โ‰กโŸจ โ‰ƒ-refl-left fe _ โŸฉ
            ฮฒ                 โˆŽ

  q = ฮป ฮณ โ†’ ฮฑ โ— (โ‰ƒ-sym ฮฑ โ— ฮณ) โ‰กโŸจ โ‰ƒ-assoc fe ฮฑ (โ‰ƒ-sym ฮฑ) ฮณ โŸฉ
            (ฮฑ โ— โ‰ƒ-sym ฮฑ) โ— ฮณ โ‰กโŸจ ap (_โ— ฮณ) (โ‰ƒ-sym-right-inverse fe ฮฑ) โŸฉ
            โ‰ƒ-refl _ โ— ฮณ      โ‰กโŸจ โ‰ƒ-refl-left fe _ โŸฉ
            ฮณ                 โˆŽ

Eq-Eq-cong : FunExt
           โ†’ {X : ๐“ค ฬ‡ } {Y : ๐“ฅ ฬ‡ } {A : ๐“ฆ ฬ‡ } {B : ๐“ฃ ฬ‡ }
           โ†’ X โ‰ƒ A โ†’ Y โ‰ƒ B โ†’ (X โ‰ƒ Y) โ‰ƒ (A โ‰ƒ B)
Eq-Eq-cong fe {X} {Y} {A} {B} ฮฑ ฮฒ =
 (X โ‰ƒ Y)  โ‰ƒโŸจ โ‰ƒ-Comp fe Y (โ‰ƒ-sym ฮฑ) โŸฉ
 (A โ‰ƒ Y)  โ‰ƒโŸจ โ‰ƒ-Sym fe โŸฉ
 (Y โ‰ƒ A)  โ‰ƒโŸจ โ‰ƒ-Comp fe A (โ‰ƒ-sym ฮฒ) โŸฉ
 (B โ‰ƒ A)  โ‰ƒโŸจ โ‰ƒ-Sym fe โŸฉ
 (A โ‰ƒ B)  โ– 

\end{code}

Propositional and functional extesionality give univalence for
propositions. Notice that P is assumed to be a proposition, but X
ranges over arbitrary types:

\begin{code}

propext-funext-give-prop-ua : propext ๐“ค โ†’ funext ๐“ค ๐“ค
                            โ†’ (X : ๐“ค ฬ‡ ) (P : ๐“ค ฬ‡ ) โ†’ is-prop P โ†’ is-equiv (idtoeq X P)
propext-funext-give-prop-ua {๐“ค} pe fe X P i = (eqtoid , ฮท) , (eqtoid , ฮต)
 where
  l : X โ‰ƒ P โ†’ is-prop X
  l e = equiv-to-prop e i
  eqtoid : X โ‰ƒ P โ†’ X โ‰ก P
  eqtoid (f , (r , rf) , h) = pe (l (f , (r , rf) , h)) i f r
  m : is-prop (X โ‰ƒ P)
  m (f , e) (f' , e') = to-ฮฃ-โ‰ก (dfunext fe (ฮป x โ†’ i (f x) (f' x)) ,
                                being-equiv-is-prop'' fe f' _ e')
  ฮท : (e : X โ‰ƒ P) โ†’ idtoeq X P (eqtoid e) โ‰ก e
  ฮท e = m (idtoeq X P (eqtoid e)) e
  ฮต : (q : X โ‰ก P) โ†’ eqtoid (idtoeq X P q) โ‰ก q
  ฮต q = identifications-of-props-are-props pe fe P i X (eqtoid (idtoeq X P q)) q

prop-univalent-โ‰ƒ : propext ๐“ค โ†’ funext ๐“ค ๐“ค โ†’ (X P : ๐“ค ฬ‡ ) โ†’ is-prop P โ†’ (X โ‰ก P) โ‰ƒ (X โ‰ƒ P)
prop-univalent-โ‰ƒ pe fe X P i = idtoeq X P , propext-funext-give-prop-ua pe fe X P i

prop-univalent-โ‰ƒ' : propext ๐“ค โ†’ funext ๐“ค ๐“ค โ†’ (X P : ๐“ค ฬ‡ ) โ†’ is-prop P โ†’ (P โ‰ก X) โ‰ƒ (P โ‰ƒ X)
prop-univalent-โ‰ƒ' pe fe X P i = (P โ‰ก X) โ‰ƒโŸจ โ‰ก-flip โŸฉ
                                (X โ‰ก P) โ‰ƒโŸจ prop-univalent-โ‰ƒ pe fe X P i โŸฉ
                                (X โ‰ƒ P) โ‰ƒโŸจ โ‰ƒ-Sym'' fe โŸฉ
                                (P โ‰ƒ X) โ– 

\end{code}

The so-called type-theoretic axiom of choice (already defined in
SpartanMLTT with another name - TODO):

\begin{code}

TT-choice : {X : ๐“ค ฬ‡ } {Y : X โ†’ ๐“ฅ ฬ‡ } {A : (x : X) โ†’ Y x โ†’ ๐“ฆ ฬ‡ }
          โ†’ (ฮ  x ๊ž‰ X , ฮฃ y ๊ž‰ Y x , A x y)
          โ†’ ฮฃ f ๊ž‰ ((x : X) โ†’ Y x) , ฮ  x ๊ž‰ X , A x (f x)
TT-choice ฯ† = (ฮป x โ†’ prโ‚(ฯ† x)) , (ฮป x โ†’ prโ‚‚(ฯ† x))

\end{code}

Its inverse (also already defined - TODO):

\begin{code}

TT-unchoice : {X : ๐“ค ฬ‡ } {Y : X โ†’ ๐“ฅ ฬ‡ } {A : (x : X) โ†’ Y x โ†’ ๐“ฆ ฬ‡ }
            โ†’ (ฮฃ f ๊ž‰ ((x : X) โ†’ Y x) , ฮ  x ๊ž‰ X , A x (f x))
            โ†’ ฮ  x ๊ž‰ X , ฮฃ y ๊ž‰ Y x , A x y
TT-unchoice (f , g) x = (f x) , (g x)

\end{code}

The proof that they are mutually inverse, where one direction requires
function extensionality (this already occurs in UF-EquivalenceExamples
- TODO):

\begin{code}

TT-choice-unchoice : {X : ๐“ค ฬ‡ } {Y : X โ†’ ๐“ฅ ฬ‡ } {A : (x : X) โ†’ Y x โ†’ ๐“ฆ ฬ‡ }
                   โ†’ (t : ฮฃ f ๊ž‰ ((x : X) โ†’ Y x) , ฮ  x ๊ž‰ X , A x (f x))
                   โ†’ TT-choice (TT-unchoice {๐“ค} {๐“ฅ} {๐“ฆ} {X} {Y} {A} t) โ‰ก t
TT-choice-unchoice t = refl

TT-choice-has-section : {X : ๐“ค ฬ‡ } {Y : X โ†’ ๐“ฅ ฬ‡ } {A : (x : X) โ†’ Y x โ†’ ๐“ฆ ฬ‡ }
                      โ†’ has-section (TT-choice {๐“ค} {๐“ฅ} {๐“ฆ} {X} {Y} {A})
TT-choice-has-section {๐“ค} {๐“ฅ} {๐“ฆ} {X} {Y} {A} = TT-unchoice ,
                                                TT-choice-unchoice {๐“ค} {๐“ฅ} {๐“ฆ} {X} {Y} {A}

TT-unchoice-choice : {X : ๐“ค ฬ‡ } {Y : X โ†’ ๐“ฅ ฬ‡ } {A : (x : X) โ†’ Y x โ†’ ๐“ฆ ฬ‡ }
                   โ†’ funext ๐“ค (๐“ฅ โŠ” ๐“ฆ)
                   โ†’ (ฯ† : ฮ  x ๊ž‰ X , ฮฃ y ๊ž‰ Y x , A x y)
                   โ†’ TT-unchoice (TT-choice ฯ†) โ‰ก ฯ†
TT-unchoice-choice fe ฯ† = dfunext fe (ฮป x โ†’ refl)

TT-choice-is-equiv : {X : ๐“ค ฬ‡ } {Y : X โ†’ ๐“ฅ ฬ‡ } {A : (x : X) โ†’ Y x โ†’ ๐“ฆ ฬ‡ }
                   โ†’ funext ๐“ค (๐“ฅ โŠ” ๐“ฆ)
                   โ†’ is-equiv TT-choice
TT-choice-is-equiv {๐“ค} {๐“ฅ} {๐“ฆ} {X} {Y} {A} fe = TT-choice-has-section {๐“ค} {๐“ฅ} {๐“ฆ} {X} {Y} {A} ,
                                                (TT-unchoice , TT-unchoice-choice fe)

TT-unchoice-is-equiv : {X : ๐“ค ฬ‡ } {Y : X โ†’ ๐“ฅ ฬ‡ } {A : (x : X) โ†’ Y x โ†’ ๐“ฆ ฬ‡ }
                     โ†’ funext ๐“ค (๐“ฅ โŠ” ๐“ฆ)
                     โ†’ is-equiv TT-unchoice
TT-unchoice-is-equiv {๐“ค} {๐“ฅ} {๐“ฆ} {X} {Y} {A} fe =
   (TT-choice , TT-unchoice-choice {๐“ค} {๐“ฅ} {๐“ฆ} {X} {Y} {A} fe) ,
   (TT-choice , TT-choice-unchoice {๐“ค} {๐“ฅ} {๐“ฆ} {X} {Y} {A})

\end{code}