Library MetaCoq.Translations.MiniHoTT_paths


Record sigT {A} (P : A Type) : Type := existT
  { projT1 : A ; projT2 : P projT1 }.

Definition sigT_ind {A} (B : A Type) (P : @sigT A B Type)
           (H : x y, P (existT _ _ x y))
  : s, P s.

Record unit : Type := tt { }.


Inductive paths (A : Type) (a : A) : A Type := idpath : paths A a a.
Definition paths_ind : A a (P : y, paths A a y Type),
    P a (idpath A a) y p, P y p.
Defined.
Definition paths_ind_beta : A a P u, paths _ (paths_ind A a P u a (idpath A a)) u.
Defined.


Notation "'exists' x .. y , p" := (sigT (fun x ⇒ .. (sigT (fun yp)) ..))
  (at level 200, x binder, right associativity,
   format "'[' 'exists' '/ ' x .. y , '/ ' p ']'")
  : type_scope.
Notation "{ x : A & P }" := (sigT (fun x:AP)) : type_scope.

Definition relation (A : Type) := A A Type.

Class Reflexive {A} (R : relation A) :=
  reflexivity : x : A, R x x.

Class Symmetric {A} (R : relation A) :=
  symmetry : x y, R x y R y x.

Class Transitive {A} (R : relation A) :=
  transitivity : x y z, R x y R y z R x z.

Class PreOrder {A} (R : relation A) :=
  { PreOrder_Reflexive : Reflexive R | 2 ;
    PreOrder_Transitive : Transitive R | 2 }.





Tactic Notation "etransitivity" open_constr(y) :=
  let R := match goal with |- ?R ?x ?zconstr:(R) end in
  let x := match goal with |- ?R ?x ?zconstr:(x) end in
  let z := match goal with |- ?R ?x ?zconstr:(z) end in
  let pre_proof_term_head := constr:(@transitivity _ R _) in
  let proof_term_head := (eval cbn in pre_proof_term_head) in
  refine (proof_term_head x y z _ _); [ change (R x y) | change (R y z) ].

Tactic Notation "etransitivity" := etransitivity _.


Notation idmap := (fun xx).



Definition const {A B} (b : B) := fun x : Ab.

Notation "( x ; y )" := (existT _ x y) : fibration_scope.
Notation pr1 := projT1.
Notation pr2 := projT2.
Notation "x .1" := (pr1 x) (at level 2, left associativity, format "x .1") : fibration_scope.
Notation "x .2" := (pr2 x) (at level 2, left associativity, format "x .2") : fibration_scope.

Notation compose := (fun g f xg (f x)).
Notation "g 'o' f" := (compose g%function f%function) (at level 40, left associativity) : function_scope.




Definition composeD {A B C} (g : b, C b) (f : A B) := fun x : Ag (f x).
Notation "g 'oD' f" := (composeD g f) (at level 40, left associativity) : function_scope.

Notation "x = y :> A" := (paths A x y) : type_scope.
Notation "x = y" := (x = y :>_) : type_scope.



Global Instance reflexive_paths {A} : Reflexive (@paths A) | 0 := @idpath A.
Notation "1" := (idpath _) : path_scope.

Definition transport {A : Type} (P : A Type) {x y : A} (p : x = y) (u : P x) : P y := paths_ind x (fun y _P y) u y p.


Definition transport_beta {A} (P : A Type) {x : A} (u : P x)
  : transport P 1 u = u
  := paths_ind_beta A x (fun y _P y) u.

Notation "p # x" := (transport _ p x) (right associativity, at level 65, only parsing) : path_scope.

Definition inverse {A : Type} {x y : A} (p : x = y) : y = x
  := transport (fun x'x' = x) p 1.

Global Instance symmetric_paths {A} : Symmetric (@paths A) | 0 := @inverse A.

Definition concat {A : Type} {x y z : A} (p : x = y) (q : y = z) : x = z.
Defined.


Global Instance transitive_paths {A} : Transitive (@paths A) | 0 := @concat A.

Notation "p @ q" := (concat p%path q%path) (at level 20) : path_scope.
Notation "p ^" := (inverse p%path) (at level 3, format "p '^'") : path_scope.

Definition ap {A B:Type} (f:A B) {x y:A} (p:x = y) : f x = f y
  := transport (fun yf x = f y) p 1.


Definition pointwise_paths {A} {P:AType} (f g: x:A, P x)
  := x:A, f x = g x.



Notation "f == g" := (pointwise_paths f g) (at level 70, no associativity) : type_scope.

Definition apD10 {A} {B:AType} {f g : x, B x} (h:f=g)
  : f == g
  := fun xtransport (fun gf x = g x) h 1.


Definition ap10 {A B} {f g:AB} (h:f=g) : f == g
  := apD10 h.


Definition ap11 {A B} {f g:AB} (h:f=g) {x y:A} (p:x=y) : f x = g y
  := ap10 h x @ ap g p.



Definition apD {A:Type} {B:AType} (f: a:A, B a) {x y:A} (p:x=y):
  p # (f x) = f y
  := paths_ind x (fun y pp # (f x) = f y) (transport_beta _ _) y p.


Definition Sect {A B : Type} (s : A B) (r : B A) :=
   x : A, r (s x) = x.


Class IsEquiv {A B : Type} (f : A B) := BuildIsEquiv {
                                               equiv_inv : B A ;
                                               eisretr : Sect equiv_inv f;
                                               eissect : Sect f equiv_inv;
                                               eisadj : x : A, eisretr (f x) = ap f (eissect x)
                                             }.


Record Equiv A B := BuildEquiv {
                        equiv_fun : A B ;
                        equiv_isequiv : IsEquiv equiv_fun
                      }.

Coercion equiv_fun : Equiv >-> Funclass.




Notation "A <~> B" := (Equiv A B) (at level 90) : type_scope.

Notation "f ^-1" := (@equiv_inv _ _ f _) (at level 3, format "f '^-1'") : function_scope.

Definition ap10_equiv {A B : Type} {f g : A <~> B} (h : f = g) : f == g
  := ap10 (ap equiv_fun h).

Class Contr (A : Type) :=
  BuildContr { center : A ;
               contr : ( y : A, center = y) }.


Class Funext := { isequiv_apD10 : (A : Type) (P : A Type) f g, IsEquiv (@apD10 A P f g) }.


Definition path_forall `{Funext} {A : Type} {P : A Type} (f g : x : A, P x) : f == g f = g
  := (@apD10 A P f g)^-1.


Definition path_forall2 `{Funext} {A B : Type} {P : A B Type} (f g : x y, P x y) :
  ( x y, f x y = g x y) f = g
  :=
    (fun Epath_forall f g (fun xpath_forall (f x) (g x) (E x))).



Definition concat_p1 {A : Type} {x y : A} (p : x = y) :
  p @ 1 = p.
Defined.

Definition concat_1p {A : Type} {x y : A} (p : x = y) :
  1 @ p = p.
Defined.

Definition concat_p_pp {A : Type} {x y z t : A} (p : x = y) (q : y = z) (r : z = t) :
  p @ (q @ r) = (p @ q) @ r.
Defined.

Definition concat_pp_p {A : Type} {x y z t : A} (p : x = y) (q : y = z) (r : z = t) :
  (p @ q) @ r = p @ (q @ r).
Defined.

Definition concat_pV {A : Type} {x y : A} (p : x = y) :
  p @ p^ = 1.
Defined.

Definition concat_Vp {A : Type} {x y : A} (p : x = y) :
  p^ @ p = 1.
Defined.

Definition concat_V_pp {A : Type} {x y z : A} (p : x = y) (q : y = z) :
  p^ @ (p @ q) = q.
Defined.

Definition concat_p_Vp {A : Type} {x y z : A} (p : x = y) (q : x = z) :
  p @ (p^ @ q) = q.
Defined.

Definition concat_pp_V {A : Type} {x y z : A} (p : x = y) (q : y = z) :
  (p @ q) @ q^ = p.
Defined.

Definition concat_pV_p {A : Type} {x y z : A} (p : x = z) (q : y = z) :
  (p @ q^) @ q = p.
Defined.

Definition inv_pp {A : Type} {x y z : A} (p : x = y) (q : y = z) :
  (p @ q)^ = q^ @ p^.
Defined.

Definition inv_Vp {A : Type} {x y z : A} (p : y = x) (q : y = z) :
  (p^ @ q)^ = q^ @ p.
Defined.

Definition inv_pV {A : Type} {x y z : A} (p : x = y) (q : z = y) :
  (p @ q^)^ = q @ p^.
Defined.

Definition inv_VV {A : Type} {x y z : A} (p : y = x) (q : z = y) :
  (p^ @ q^)^ = q @ p.
Defined.

Definition inv_V {A : Type} {x y : A} (p : x = y) :
  p^^ = p.
Defined.

Definition moveR_Mp {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : y = x) :
  p = r^ @ q r @ p = q.

Definition moveR_pM {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : y = x) :
  r = q @ p^ r @ p = q.

Definition moveR_Vp {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : x = y) :
  p = r @ q r^ @ p = q.

Definition moveR_pV {A : Type} {x y z : A} (p : z = x) (q : y = z) (r : y = x) :
  r = q @ p r @ p^ = q.

Definition moveL_Mp {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : y = x) :
  r^ @ q = p q = r @ p.

Definition moveL_pM {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : y = x) :
  q @ p^ = r q = r @ p.

Definition moveL_Vp {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : x = y) :
  r @ q = p q = r^ @ p.

Definition moveL_pV {A : Type} {x y z : A} (p : z = x) (q : y = z) (r : y = x) :
  q @ p = r q = r @ p^.

Definition moveL_1M {A : Type} {x y : A} (p q : x = y) :
  p @ q^ = 1 p = q.

Definition moveL_M1 {A : Type} {x y : A} (p q : x = y) :
  q^ @ p = 1 p = q.

Definition moveL_1V {A : Type} {x y : A} (p : x = y) (q : y = x) :
  p @ q = 1 p = q^.

Definition moveL_V1 {A : Type} {x y : A} (p : x = y) (q : y = x) :
  q @ p = 1 p = q^.

Definition moveR_M1 {A : Type} {x y : A} (p q : x = y) :
  1 = p^ @ q p = q.

Definition moveR_1M {A : Type} {x y : A} (p q : x = y) :
  1 = q @ p^ p = q.

Definition moveR_1V {A : Type} {x y : A} (p : x = y) (q : y = x) :
  1 = q @ p p^ = q.

Definition moveR_V1 {A : Type} {x y : A} (p : x = y) (q : y = x) :
  1 = p @ q p^ = q.

Definition moveR_transport_p {A : Type} (P : A Type) {x y : A}
  (p : x = y) (u : P x) (v : P y)
  : u = p^ # v p # u = v.

Definition moveR_transport_V {A : Type} (P : A Type) {x y : A}
  (p : y = x) (u : P x) (v : P y)
  : u = p # v p^ # u = v.

Definition moveL_transport_V {A : Type} (P : A Type) {x y : A}
  (p : x = y) (u : P x) (v : P y)
  : p # u = v u = p^ # v.

Definition moveL_transport_p {A : Type} (P : A Type) {x y : A}
  (p : y = x) (u : P x) (v : P y)
  : p^ # u = v u = p # v.

Definition moveR_transport_p_V {A : Type} (P : A Type) {x y : A}
           (p : x = y) (u : P x) (v : P y) (q : u = p^ # v)
  : (moveR_transport_p P p u v q)^ = moveL_transport_p P p v u q^.

Definition moveR_transport_V_V {A : Type} (P : A Type) {x y : A}
           (p : y = x) (u : P x) (v : P y) (q : u = p # v)
  : (moveR_transport_V P p u v q)^ = moveL_transport_V P p v u q^.

Definition moveL_transport_V_V {A : Type} (P : A Type) {x y : A}
           (p : x = y) (u : P x) (v : P y) (q : p # u = v)
  : (moveL_transport_V P p u v q)^ = moveR_transport_V P p v u q^.

Definition moveL_transport_p_V {A : Type} (P : A Type) {x y : A}
           (p : y = x) (u : P x) (v : P y) (q : p^ # u = v)
  : (moveL_transport_p P p u v q)^ = moveR_transport_p P p v u q^.

Definition ap_1 {A B : Type} (x : A) (f : A B) :
  ap f 1 = 1 :> (f x = f x)
  := 1.

Definition apD_1 {A B} (x : A) (f : x : A, B x) :
  apD f 1 = 1 :> (f x = f x)
  := 1.

Definition ap_pp {A B : Type} (f : A B) {x y z : A} (p : x = y) (q : y = z) :
  ap f (p @ q) = (ap f p) @ (ap f q).
Defined.

Definition ap_p_pp {A B : Type} (f : A B) {w : B} {x y z : A}
  (r : w = f x) (p : x = y) (q : y = z) :
  r @ (ap f (p @ q)) = (r @ ap f p) @ (ap f q).

Definition ap_pp_p {A B : Type} (f : A B) {x y z : A} {w : B}
  (p : x = y) (q : y = z) (r : f z = w) :
  (ap f (p @ q)) @ r = (ap f p) @ (ap f q @ r).

Definition inverse_ap {A B : Type} (f : A B) {x y : A} (p : x = y) :
  (ap f p)^ = ap f (p^).
Defined.

Definition ap_V {A B : Type} (f : A B) {x y : A} (p : x = y) :
  ap f (p^) = (ap f p)^.
Defined.

Definition ap_idmap {A : Type} {x y : A} (p : x = y) :
  ap idmap p = p.
Defined.

Definition ap_compose {A B C : Type} (f : A B) (g : B C) {x y : A} (p : x = y) :
  ap (g o f) p = ap g (ap f p).
Defined.

Definition ap_compose' {A B C : Type} (f : A B) (g : B C) {x y : A} (p : x = y) :
  ap (fun ag (f a)) p = ap g (ap f p).
Defined.

Definition ap_const {A B : Type} {x y : A} (p : x = y) (z : B) :
  ap (fun _z) p = 1.
Defined.

Definition concat_Ap {A B : Type} {f g : A B} (p : x, f x = g x) {x y : A} (q : x = y) :
  (ap f q) @ (p y) = (p x) @ (ap g q).
Defined.

Definition concat_A1p {A : Type} {f : A A} (p : x, f x = x) {x y : A} (q : x = y) :
  (ap f q) @ (p y) = (p x) @ q.
Defined.

Definition concat_pA1 {A : Type} {f : A A} (p : x, x = f x) {x y : A} (q : x = y) :
  (p x) @ (ap f q) = q @ (p y).
Defined.

Definition concat_pA_pp {A B : Type} {f g : A B} (p : x, f x = g x)
  {x y : A} (q : x = y)
  {w z : B} (r : w = f x) (s : g y = z)
  :
  (r @ ap f q) @ (p y @ s) = (r @ p x) @ (ap g q @ s).

Definition concat_pA_p {A B : Type} {f g : A B} (p : x, f x = g x)
  {x y : A} (q : x = y)
  {w : B} (r : w = f x)
  :
  (r @ ap f q) @ p y = (r @ p x) @ ap g q.

Definition concat_A_pp {A B : Type} {f g : A B} (p : x, f x = g x)
  {x y : A} (q : x = y)
  {z : B} (s : g y = z)
  :
  (ap f q) @ (p y @ s) = (p x) @ (ap g q @ s).

Definition concat_pA1_pp {A : Type} {f : A A} (p : x, f x = x)
  {x y : A} (q : x = y)
  {w z : A} (r : w = f x) (s : y = z)
  :
  (r @ ap f q) @ (p y @ s) = (r @ p x) @ (q @ s).

Definition concat_pp_A1p {A : Type} {g : A A} (p : x, x = g x)
  {x y : A} (q : x = y)
  {w z : A} (r : w = x) (s : g y = z)
  :
  (r @ p x) @ (ap g q @ s) = (r @ q) @ (p y @ s).

Definition concat_pA1_p {A : Type} {f : A A} (p : x, f x = x)
  {x y : A} (q : x = y)
  {w : A} (r : w = f x)
  :
  (r @ ap f q) @ p y = (r @ p x) @ q.

Definition concat_A1_pp {A : Type} {f : A A} (p : x, f x = x)
  {x y : A} (q : x = y)
  {z : A} (s : y = z)
  :
  (ap f q) @ (p y @ s) = (p x) @ (q @ s).

Definition concat_pp_A1 {A : Type} {g : A A} (p : x, x = g x)
  {x y : A} (q : x = y)
  {w : A} (r : w = x)
  :
  (r @ p x) @ ap g q = (r @ q) @ p y.

Definition concat_p_A1p {A : Type} {g : A A} (p : x, x = g x)
  {x y : A} (q : x = y)
  {z : A} (s : g y = z)
  :
  p x @ (ap g q @ s) = q @ (p y @ s).

Lemma concat_1p_1 {A} {x : A} (p : x = x) (q : p = 1)
: concat_1p p @ q = ap (fun p' ⇒ 1 @ p') q.

Lemma concat_p1_1 {A} {x : A} (p : x = x) (q : p = 1)
: concat_p1 p @ q = ap (fun p'p' @ 1) q.

Definition apD10_1 {A} {B:AType} (f : x, B x) (x:A)
  : apD10 (idpath f) x = 1
:= 1.

Definition apD10_pp {A} {B:AType} {f f' f'' : x, B x}
  (h:f=f') (h':f'=f'') (x:A)
: apD10 (h @ h') x = apD10 h x @ apD10 h' x.

Definition apD10_V {A} {B:AType} {f g : x, B x} (h:f=g) (x:A)
  : apD10 (h^) x = (apD10 h x)^.
Defined.

Definition ap10_1 {A B} {f:AB} (x:A) : ap10 (idpath f) x = 1
  := 1.

Definition ap10_pp {A B} {f f' f'':AB} (h:f=f') (h':f'=f'') (x:A)
  : ap10 (h @ h') x = ap10 h x @ ap10 h' x
:= apD10_pp h h' x.

Definition ap10_V {A B} {f g : AB} (h : f = g) (x:A)
  : ap10 (h^) x = (ap10 h x)^
:= apD10_V h x.

Definition apD10_ap_precompose {A B C} (f : A B) {g g' : x:B, C x} (p : g = g') a
: apD10 (ap (fun h : x:B, C xh oD f) p) a = apD10 p (f a).

Definition ap10_ap_precompose {A B C} (f : A B) {g g' : B C} (p : g = g') a
: ap10 (ap (fun h : B Ch o f) p) a = ap10 p (f a)
  := apD10_ap_precompose f p a.

Definition apD10_ap_postcompose {A B C} (f : x, B x C) {g g' : x:A, B x} (p : g = g') a
: apD10 (ap (fun h : x:A, B xfun xf x (h x)) p) a = ap (f a) (apD10 p a).

Definition ap10_ap_postcompose {A B C} (f : B C) {g g' : A B} (p : g = g') a
: ap10 (ap (fun h : A Bf o h) p) a = ap f (ap10 p a)
:= apD10_ap_postcompose (fun af) p a.

Definition transport_1 {A : Type} (P : A Type) {x : A} (u : P x)
  : 1 # u = u
:= 1.

Definition transport_pp {A : Type} (P : A Type) {x y z : A} (p : x = y) (q : y = z) (u : P x) :
  p @ q # u = q # p # u.
Defined.

Definition transport_pV {A : Type} (P : A Type) {x y : A} (p : x = y) (z : P y)
  : p # p^ # z = z
  := (transport_pp P p^ p z)^
  @ ap (fun rtransport P r z) (concat_Vp p).

Definition transport_Vp {A : Type} (P : A Type) {x y : A} (p : x = y) (z : P x)
  : p^ # p # z = z
  := (transport_pp P p p^ z)^
  @ ap (fun rtransport P r z) (concat_pV p).

Definition transport_p_pp {A : Type} (P : A Type)
  {x y z w : A} (p : x = y) (q : y = z) (r : z = w)
  (u : P x)
  : ap (fun ee # u) (concat_p_pp p q r)
    @ (transport_pp P (p@q) r u) @ ap (transport P r) (transport_pp P p q u)
  = (transport_pp P p (q@r) u) @ (transport_pp P q r (p#u))
  :> ((p @ (q @ r)) # u = r # q # p # u) .

Definition transport_pVp {A} (P : A Type) {x y:A} (p:x=y) (z:P x)
  : transport_pV P p (transport P p z)
  = ap (transport P p) (transport_Vp P p z).

Definition transport_VpV {A} (P : A Type) {x y : A} (p : x = y) (z : P y)
  : transport_Vp P p (transport P p^ z)
    = ap (transport P p^) (transport_pV P p z).

Definition ap_transport_transport_pV {A} (P : A Type) {x y : A}
           (p : x = y) (u : P x) (v : P y) (e : transport P p u = v)
  : ap (transport P p) (moveL_transport_V P p u v e)
       @ transport_pV P p v = e.

Definition moveL_transport_V_1 {A} (P : A Type) {x y : A}
           (p : x = y) (u : P x)
  : moveL_transport_V P p u (p # u) 1 = (transport_Vp P p u)^.

Definition ap11_is_ap10_ap01 {A B} {f g:AB} (h:f=g) {x y:A} (p:x=y)
: ap11 h p = ap10 h x @ ap g p.
Defined.

Definition transportD {A : Type} (B : A Type) (C : a:A, B a Type)
  {x1 x2 : A} (p : x1 = x2) (y : B x1) (z : C x1 y)
  : C x2 (p # y).
Defined.

Definition transportD2 {A : Type} (B C : A Type) (D : a:A, B a C a Type)
  {x1 x2 : A} (p : x1 = x2) (y : B x1) (z : C x1) (w : D x1 y z)
  : D x2 (p # y) (p # z).
Defined.

Definition ap011 {A B C} (f : A B C) {x x' y y'} (p : x = x') (q : y = y')
: f x y = f x' y'
:= ap11 (ap f p) q.

Definition ap011D {A B C} (f : (a:A), B a C)
           {x x'} (p : x = x') {y y'} (q : p # y = y')
: f x y = f x' y'.

Definition ap01D1 {A B C} (f : (a:A), B a C a)
           {x x'} (p : x = x') {y y'} (q : p # y = y')
: transport C p (f x y) = f x' y'.

Definition apD011 {A B C} (f : (a:A) (b:B a), C a b)
           {x x'} (p : x = x') {y y'} (q : p # y = y')
: transport (C x') q (transportD B C p y (f x y)) = f x' y'.

Definition transport2 {A : Type} (P : A Type) {x y : A} {p q : x = y}
  (r : p = q) (z : P x)
  : p # z = q # z
  := ap (fun p'p' # z) r.

Definition transport2_is_ap10 {A : Type} (Q : A Type) {x y : A} {p q : x = y}
  (r : p = q) (z : Q x)
  : transport2 Q r z = ap10 (ap (transport Q) r) z.
Defined.

Definition transport2_p2p {A : Type} (P : A Type) {x y : A} {p1 p2 p3 : x = y}
  (r1 : p1 = p2) (r2 : p2 = p3) (z : P x)
  : transport2 P (r1 @ r2) z = transport2 P r1 z @ transport2 P r2 z.

Definition transport2_V {A : Type} (Q : A Type) {x y : A} {p q : x = y}
  (r : p = q) (z : Q x)
  : transport2 Q (r^) z = (transport2 Q r z)^.
Defined.

Definition concat_AT {A : Type} (P : A Type) {x y : A} {p q : x = y}
  {z w : P x} (r : p = q) (s : z = w)
  : ap (transport P p) s @ transport2 P r w
    = transport2 P r z @ ap (transport P q) s.
Defined.

Lemma ap_transport {A} {P Q : A Type} {x y : A} (p : x = y) (f : x, P x Q x) (z : P x) :
  f y (p # z) = (p # (f x z)).

Lemma ap_transportD {A : Type}
      (B : A Type) (C1 C2 : a : A, B a Type)
      (f : a b, C1 a b C2 a b)
      {x1 x2 : A} (p : x1 = x2) (y : B x1) (z : C1 x1 y)
: f x2 (p # y) (transportD B C1 p y z)
  = transportD B C2 p y (f x1 y z).

Lemma ap_transportD2 {A : Type}
      (B C : A Type) (D1 D2 : a, B a C a Type)
      (f : a b c, D1 a b c D2 a b c)
      {x1 x2 : A} (p : x1 = x2) (y : B x1) (z : C x1) (w : D1 x1 y z)
: f x2 (p # y) (p # z) (transportD2 B C D1 p y z w)
  = transportD2 B C D2 p y z (f x1 y z w).

Lemma ap_transport_pV {X} (Y : X Type) {x1 x2 : X} (p : x1 = x2)
      {y1 y2 : Y x2} (q : y1 = y2)
: ap (transport Y p) (ap (transport Y p^) q) =
  transport_pV Y p y1 @ q @ (transport_pV Y p y2)^.

Definition transport_pV_ap {X} (P : X Type) (f : x, P x)
      {x1 x2 : X} (p : x1 = x2)
: ap (transport P p) (apD f p^) @ apD f p = transport_pV P p (f x2).

Definition apD_pp {A} {P : A Type} (f : x, P x)
           {x y z : A} (p : x = y) (q : y = z)
  : apD f (p @ q)
    = transport_pp P p q (f x) @ ap (transport P q) (apD f p) @ apD f q.

Definition apD_V {A} {P : A Type} (f : x, P x)
           {x y : A} (p : x = y)
  : apD f p^ = moveR_transport_V _ _ _ _ (apD f p)^.
Definition transport_const {A B : Type} {x1 x2 : A} (p : x1 = x2) (y : B)
  : transport (fun xB) p y = y.

Definition transport2_const {A B : Type} {x1 x2 : A} {p q : x1 = x2}
  (r : p = q) (y : B)
  : transport_const p y = transport2 (fun _B) r y @ transport_const q y.
Defined.

Lemma transport_compose {A B} {x y : A} (P : B Type) (f : A B)
  (p : x = y) (z : P (f x))
  : transport (fun xP (f x)) p z = transport P (ap f p) z.

Lemma transportD_compose {A A'} B {x x' : A} (C : x : A', B x Type) (f : A A')
      (p : x = x') y (z : C (f x) y)
: transportD (B o f) (C oD f) p y z
  = transport (C (f x')) (transport_compose B f p y)^ (transportD B C (ap f p) y z).

Lemma transport_apD_transportD {A} B (f : x : A, B x) (C : x, B x Type)
      {x1 x2 : A} (p : x1 = x2) (z : C x1 (f x1))
: apD f p # transportD B C p _ z
  = transport (fun xC x (f x)) p z.

Lemma transport_precompose {A B C} (f : A B) (g g' : B C) (p : g = g')
: transport (fun h : B Cg o f = h o f) p 1 =
  ap (fun hh o f) p.

Definition transport_idmap_ap A (P : A Type) x y (p : x = y) (u : P x)
: transport P p u = transport idmap (ap P p) u.
Defined.

Sometimes, it's useful to have the goal be in terms of ap, so we can use lemmas about ap. However, we can't just rewrite !transport_idmap_ap, as that's likely to loop. So, instead, we provide a tactic transport_to_ap, that replaces all transport P p u with transport idmap (ap P p) u for non-idmap P.

Definition transport_transport {A B} (C : A B Type)
           {x1 x2 : A} (p : x1 = x2) {y1 y2 : B} (q : y1 = y2)
           (c : C x1 y1)
: transport (C x2) q (transport (fun xC x y1) p c)
  = transport (fun xC x y2) p (transport (C x1) q c).

Lemma apD_const {A B} {x y : A} (f : A B) (p: x = y) :
  apD f p = transport_const p (f x) @ ap f p.

Definition concat2 {A} {x y z : A} {p p' : x = y} {q q' : y = z} (h : p = p') (h' : q = q')
  : p @ q = p' @ q'.
Defined.

Notation "p @@ q" := (concat2 p q)%path (at level 20) : path_scope.


Lemma concat2_ap_ap {A B : Type} {x' y' z' : B}
           (f : A (x' = y')) (g : A (y' = z'))
           {x y : A} (p : x = y)
: (ap f p) @@ (ap g p) = ap (fun uf u @ g u) p.

Definition inverse2 {A : Type} {x y : A} {p q : x = y} (h : p = q)
  : p^ = q^
:= ap inverse h.

Lemma ap_pp_concat_pV {A B} (f : A B) {x y : A} (p : x = y)
: ap_pp f p p^ @ ((1 @@ ap_V f p) @ concat_pV (ap f p))
  = ap (ap f) (concat_pV p).

Lemma ap_pp_concat_Vp {A B} (f : A B) {x y : A} (p : x = y)
: ap_pp f p^ p @ ((ap_V f p @@ 1) @ concat_Vp (ap f p))
  = ap (ap f) (concat_Vp p).

Lemma concat_pV_inverse2 {A} {x y : A} (p q : x = y) (r : p = q)
: (r @@ inverse2 r) @ concat_pV q = concat_pV p.

Lemma concat_Vp_inverse2 {A} {x y : A} (p q : x = y) (r : p = q)
: (inverse2 r @@ r) @ concat_Vp q = concat_Vp p.

Definition whiskerL {A : Type} {x y z : A} (p : x = y)
  {q r : y = z} (h : q = r) : p @ q = p @ r
:= 1 @@ h.

Definition whiskerR {A : Type} {x y z : A} {p q : x = y}
  (h : p = q) (r : y = z) : p @ r = q @ r
:= h @@ 1.

Definition cancelL {A} {x y z : A} (p : x = y) (q r : y = z)
: (p @ q = p @ r) (q = r)
:= fun h(concat_V_pp p q)^ @ whiskerL p^ h @ (concat_V_pp p r).

Definition cancelR {A} {x y z : A} (p q : x = y) (r : y = z)
: (p @ r = q @ r) (p = q)
:= fun h(concat_pp_V p r)^ @ whiskerR h r^ @ (concat_pp_V q r).

Definition whiskerR_p1 {A : Type} {x y : A} {p q : x = y} (h : p = q) :
  (concat_p1 p) ^ @ whiskerR h 1 @ concat_p1 q = h.
Defined.

Definition whiskerR_1p {A : Type} {x y z : A} (p : x = y) (q : y = z) :
  whiskerR 1 q = 1 :> (p @ q = p @ q).
Defined.

Definition whiskerL_p1 {A : Type} {x y z : A} (p : x = y) (q : y = z) :
  whiskerL p 1 = 1 :> (p @ q = p @ q).
Defined.

Definition whiskerL_1p {A : Type} {x y : A} {p q : x = y} (h : p = q) :
  (concat_1p p) ^ @ whiskerL 1 h @ concat_1p q = h.
Defined.

Definition whiskerR_p1_1 {A} {x : A} (h : idpath x = idpath x)
: whiskerR h 1 = h.

Definition whiskerL_1p_1 {A} {x : A} (h : idpath x = idpath x)
: whiskerL 1 h = h.

Definition concat2_p1 {A : Type} {x y : A} {p q : x = y} (h : p = q) :
  h @@ 1 = whiskerR h 1 :> (p @ 1 = q @ 1).
Defined.

Definition concat2_1p {A : Type} {x y : A} {p q : x = y} (h : p = q) :
  1 @@ h = whiskerL 1 h :> (1 @ p = 1 @ q).
Defined.

Definition cancel2L {A : Type} {x y z : A} {p p' : x = y} {q q' : y = z}
           (g : p = p') (h k : q = q')
: (g @@ h = g @@ k) (h = k).

Definition cancel2R {A : Type} {x y z : A} {p p' : x = y} {q q' : y = z}
           (g h : p = p') (k : q = q')
: (g @@ k = h @@ k) (g = h).

Definition whiskerL_pp {A} {x y z : A} (p : x = y) {q q' q'' : y = z}
           (r : q = q') (s : q' = q'')
: whiskerL p (r @ s) = whiskerL p r @ whiskerL p s.

Definition whiskerR_pp {A} {x y z : A} {p p' p'' : x = y} (q : y = z)
           (r : p = p') (s : p' = p'')
: whiskerR (r @ s) q = whiskerR r q @ whiskerR s q.

Definition whiskerL_VpL {A} {x y z : A} (p : x = y)
           {q q' : y = z} (r : q = q')
: (concat_V_pp p q)^ @ whiskerL p^ (whiskerL p r) @ concat_V_pp p q'
  = r.

Definition whiskerL_pVL {A} {x y z : A} (p : y = x)
           {q q' : y = z} (r : q = q')
: (concat_p_Vp p q)^ @ whiskerL p (whiskerL p^ r) @ concat_p_Vp p q'
  = r.

Definition whiskerR_pVR {A} {x y z : A} {p p' : x = y}
           (r : p = p') (q : y = z)
: (concat_pp_V p q)^ @ whiskerR (whiskerR r q) q^ @ concat_pp_V p' q
  = r.

Definition whiskerR_VpR {A} {x y z : A} {p p' : x = y}
           (r : p = p') (q : z = y)
: (concat_pV_p p q)^ @ whiskerR (whiskerR r q^) q @ concat_pV_p p' q
  = r.

Definition concat_concat2 {A : Type} {x y z : A} {p p' p'' : x = y} {q q' q'' : y = z}
  (a : p = p') (b : p' = p'') (c : q = q') (d : q' = q'') :
  (a @@ c) @ (b @@ d) = (a @ b) @@ (c @ d).

Definition concat_whisker {A} {x y z : A} (p p' : x = y) (q q' : y = z) (a : p = p') (b : q = q') :
  (whiskerR a q) @ (whiskerL p' b) = (whiskerL p b) @ (whiskerR a q').
Defined.

Definition pentagon {A : Type} {v w x y z : A} (p : v = w) (q : w = x) (r : x = y) (s : y = z)
  : whiskerL p (concat_p_pp q r s)
      @ concat_p_pp p (q@r) s
      @ whiskerR (concat_p_pp p q r) s
  = concat_p_pp p q (r@s) @ concat_p_pp (p@q) r s.

Definition triangulator {A : Type} {x y z : A} (p : x = y) (q : y = z)
  : concat_p_pp p 1 q @ whiskerR (concat_p1 p) q
  = whiskerL p (concat_1p q).

Definition eckmann_hilton {A : Type} {x:A} (p q : 1 = 1 :> (x = x)) : p @ q = q @ p :=
  (whiskerR_p1 p @@ whiskerL_1p q)^
  @ (concat_p1 _ @@ concat_p1 _)
  @ (concat_1p _ @@ concat_1p _)
  @ (concat_whisker _ _ _ _ p q)
  @ (concat_1p _ @@ concat_1p _)^
  @ (concat_p1 _ @@ concat_p1 _)^
  @ (whiskerL_1p q @@ whiskerR_p1 p).

Definition ap02 {A B : Type} (f:AB) {x y:A} {p q:x=y} (r:p=q) : ap f p = ap f q.
Defined.

Definition ap02_pp {A B} (f:AB) {x y:A} {p p' p'':x=y} (r:p=p') (r':p'=p'')
  : ap02 f (r @ r') = ap02 f r @ ap02 f r'.

Definition ap02_p2p {A B} (f:AB) {x y z:A} {p p':x=y} {q q':y=z} (r:p=p') (s:q=q')
  : ap02 f (r @@ s) = ap_pp f p q
                      @ (ap02 f r @@ ap02 f s)
                      @ (ap_pp f p' q')^.

Definition apD02 {A : Type} {B : A Type} {x y : A} {p q : x = y}
  (f : x, B x) (r : p = q)
  : apD f p = transport2 B r (f x) @ apD f q.
Defined.

Definition apD02_const {A B : Type} (f : A B) {x y : A} {p q : x = y} (r : p = q)
: apD02 f r = (apD_const f p)
              @ (transport2_const r (f x) @@ ap02 f r)
              @ (concat_p_pp _ _ _)^
              @ (whiskerL (transport2 _ r (f x)) (apD_const f q)^).
Defined.

Definition apD02_pp {A} (B : A Type) (f : x:A, B x) {x y : A}
  {p1 p2 p3 : x = y} (r1 : p1 = p2) (r2 : p2 = p3)
  : apD02 f (r1 @ r2)
  = apD02 f r1
  @ whiskerL (transport2 B r1 (f x)) (apD02 f r2)
  @ concat_p_pp _ _ _
  @ (whiskerR (transport2_p2p B r1 r2 (f x))^ (apD f p3)).

Definition ap_transport_Vp_idmap {A B} (p q : A = B) (r : q = p) (z : A)
: ap (transport idmap q^) (ap (fun stransport idmap s z) r)
  @ ap (fun stransport idmap s (p # z)) (inverse2 r)
  @ transport_Vp idmap p z
  = transport_Vp idmap q z.

Definition ap_transport_pV_idmap {A B} (p q : A = B) (r : q = p) (z : B)
: ap (transport idmap q) (ap (fun stransport idmap s^ z) r)
  @ ap (fun stransport idmap s (p^ # z)) r
  @ transport_pV idmap p z
  = transport_pV idmap q z.

Notation concatR := (fun p qconcat q p).





If a space is contractible, then any two points in it are connected by a path in a canonical way.
Definition path_contr `{Contr A} (x y : A) : x = y
  := (contr x)^ @ (contr y).

Similarly, any two parallel paths in a contractible space are homotopic, which is just the principle UIP.
Definition path2_contr `{Contr A} {x y : A} (p q : x = y) : p = q.

It follows that any space of paths in a contractible space is contractible. Because Contr is a notation, and Contr_internal is the record, we need to iota expand to fool Coq's typeclass machinery into accepting supposedly "mismatched" contexts.

Global Instance contr_paths_contr `{Contr A} (x y : A) : Contr (x = y) | 10000 := let c := {|
  center := (contr x)^ @ contr y;
  contr := path2_contr ((contr x)^ @ contr y)
|} in c.

Also, the total space of any based path space is contractible. We define the contr fields as separate definitions, so that we can give them simpl nomatch annotations.

Definition path_basedpaths {X : Type} {x y : X} (p : x = y)
: (x;1) = (y;p) :> {z:X & x=z}.


Global Instance contr_basedpaths {X : Type} (x : X) : Contr {y : X & x = y} | 100.

Definition path_basedpaths' {X : Type} {x y : X} (p : y = x)
: @existT _ (fun z ⇒ @paths X z x) x 1 = (y; p).

Global Instance contr_basedpaths' {X : Type} (x : X) : Contr {y : X & y = x} | 100.


Definition ap_pr1_path_contr_basedpaths {X : Type}
           {x y z : X} (p : x = y) (q : x = z)
: ap pr1 (path_contr ((y;p):{y':X & x = y'}) (z;q)) = p^ @ q.

Definition ap_pr1_path_contr_basedpaths' {X : Type}
           {x y z : X} (p : y = x) (q : z = x)
: ap pr1 (path_contr ((y;p):{y':X & y' = x}) (z;q)) = p @ q^.

Definition ap_pr1_path_basedpaths {X : Type}
           {x y : X} (p : x = y)
: ap pr1 (path_basedpaths p) = p.

Definition ap_pr1_path_basedpaths' {X : Type}
           {x y : X} (p : y = x)
: ap pr1 (path_basedpaths' p) = p^.

If the domain is contractible, the function is propositionally constant.
Definition contr_dom_equiv {A B} (f : A B) `{Contr A} : x y : A, f x = f y
  := fun x yap f ((contr x)^ @ contr y).


Global Instance isequiv_idmap (A : Type) : IsEquiv idmap | 0 :=
  BuildIsEquiv A A idmap idmap (fun _ ⇒ 1) (fun _ ⇒ 1) (fun _ ⇒ 1).

Definition equiv_idmap (A : Type) : A <~> A := BuildEquiv A A idmap _.


Notation "1" := equiv_idmap : equiv_scope.

Global Instance reflexive_equiv : Reflexive Equiv | 0 := @equiv_idmap.

The composition of equivalences is an equivalence.
Global Instance isequiv_compose `{IsEquiv A B f} `{IsEquiv B C g}
  : IsEquiv (compose g f) | 1000
  := BuildIsEquiv A C (compose g f)
    (compose f^-1 g^-1)
    (fun cap g (eisretr f (g^-1 c)) @ eisretr g c)
    (fun aap (f^-1) (eissect g (f a)) @ eissect f a)
    (fun a
      (whiskerL _ (eisadj g (f a))) @
      (ap_pp g _ _)^ @
      ap02 g
      ( (concat_A1p (eisretr f) (eissect g (f a)))^ @
        (ap_compose f^-1 f _ @@ eisadj f a) @
        (ap_pp f _ _)^
      ) @
      (ap_compose f g _)^
    ).

Definition isequiv_compose'
  {A B : Type} (f : A B) (_ : IsEquiv f)
  {C : Type} (g : B C) (_ : IsEquiv g)
  : IsEquiv (g o f)
  := isequiv_compose.

Definition equiv_compose {A B C : Type} (g : B C) (f : A B)
  `{IsEquiv B C g} `{IsEquiv A B f}
  : A <~> C
  := BuildEquiv A C (compose g f) _.

Definition equiv_compose' {A B C : Type} (g : B <~> C) (f : A <~> B)
  : A <~> C
  := equiv_compose g f.

We put g and f in equiv_scope explcitly. This is a partial work-around for https://coq.inria.fr/bugs/show_bug.cgi?id=3990, which is that implicitly bound scopes don't nest well.
Notation "g 'oE' f" := (equiv_compose' g%equiv f%equiv) (at level 40, left associativity) : equiv_scope.

Global Instance transitive_equiv : Transitive Equiv | 0 :=
  fun _ _ _ f gequiv_compose g f.

Anything homotopic to an equivalence is an equivalence.
Section IsEquivHomotopic.

  Context {A B : Type} (f : A B) {g : A B}.
  Context `{IsEquiv A B f}.
  Hypothesis h : f == g.

  Let sect := (fun b:B(h (f^-1 b))^ @ eisretr f b).
  Let retr := (fun a:A(ap f^-1 (h a))^ @ eissect f a).

  Let adj (a : A) : sect (g a) = ap g (retr a).

  Definition isequiv_homotopic : IsEquiv g
    := BuildIsEquiv _ _ g (f ^-1) sect retr adj.

  Definition equiv_homotopic : A <~> B
    := BuildEquiv _ _ g isequiv_homotopic.

End IsEquivHomotopic.

The inverse of an equivalence is an equivalence.
Section EquivInverse.

  Context {A B : Type} (f : A B) {feq : IsEquiv f}.

  Theorem other_adj (b : B) : eissect f (f^-1 b) = ap f^-1 (eisretr f b).

  Global Instance isequiv_inverse : IsEquiv f^-1 | 10000
    := BuildIsEquiv B A f^-1 f (eissect f) (eisretr f) other_adj.
End EquivInverse.

If the goal is IsEquiv _^-1, then use isequiv_inverse; otherwise, don't pretend worry about if the goal is an evar and we want to add a ^-1.

Equiv A B is a symmetric relation.
Theorem equiv_inverse {A B : Type} : (A <~> B) (B <~> A).

Notation "e ^-1" := (@equiv_inverse _ _ e) : equiv_scope.

Global Instance symmetric_equiv : Symmetric Equiv | 0 := @equiv_inverse.

If g \o f and f are equivalences, so is g. This is not an Instance because it would require Coq to guess f.
Definition cancelR_isequiv {A B C} (f : A B) {g : B C}
  `{IsEquiv A B f} `{IsEquiv A C (g o f)}
  : IsEquiv g
  := isequiv_homotopic (compose (compose g f) f^-1)
       (fun bap g (eisretr f b)).

Definition cancelR_equiv {A B C} (f : A B) {g : B C}
  `{IsEquiv A B f} `{IsEquiv A C (g o f)}
  : B <~> C
  := BuildEquiv B C g (cancelR_isequiv f).

If g \o f and g are equivalences, so is f.
Definition cancelL_isequiv {A B C} (g : B C) {f : A B}
  `{IsEquiv B C g} `{IsEquiv A C (g o f)}
  : IsEquiv f
  := isequiv_homotopic (compose g^-1 (compose g f))
       (fun aeissect g (f a)).

Definition cancelL_equiv {A B C} (g : B C) {f : A B}
  `{IsEquiv B C g} `{IsEquiv A C (g o f)}
  : A <~> B
  := BuildEquiv _ _ f (cancelL_isequiv g).

Combining these with isequiv_compose, we see that equivalences can be transported across commutative squares.
Definition isequiv_commsq {A B C D}
           (f : A B) (g : C D) (h : A C) (k : B D)
           (p : k o f == g o h)
           `{IsEquiv _ _ f} `{IsEquiv _ _ h} `{IsEquiv _ _ k}
: IsEquiv g.

Definition isequiv_commsq' {A B C D}
           (f : A B) (g : C D) (h : A C) (k : B D)
           (p : g o h == k o f)
           `{IsEquiv _ _ g} `{IsEquiv _ _ h} `{IsEquiv _ _ k}
: IsEquiv f.

Transporting is an equivalence.
Section EquivTransport.

  Context {A : Type} (P : A Type) (x y : A) (p : x = y).

  Global Instance isequiv_transport : IsEquiv (transport P p) | 0
    := BuildIsEquiv (P x) (P y) (transport P p) (transport P p^)
    (transport_pV P p) (transport_Vp P p) (transport_pVp P p).

  Definition equiv_transport : P x <~> P y
    := BuildEquiv _ _ (transport P p) _.

End EquivTransport.

In all the above cases, we were able to directly construct all the structure of an equivalence. However, as is evident, sometimes it is quite difficult to prove the adjoint law.
The following adjointification theorem allows us to be lazy about this if we wish. It says that if we have all the data of an (adjoint) equivalence except the triangle identity, then we can always obtain the triangle identity by modifying the datum equiv_is_section (or equiv_is_retraction). The proof is the same as the standard categorical argument that any equivalence can be improved to an adjoint equivalence.
As a stylistic matter, we try to avoid using adjointification in the library whenever possible, to preserve the homotopies specified by the user.

Section Adjointify.

  Context {A B : Type} (f : A B) (g : B A).
  Context (isretr : Sect g f) (issect : Sect f g).

  Let issect' := fun x
    ap g (ap f (issect x)^) @ ap g (isretr (f x)) @ issect x.

  Let is_adjoint' (a : A) : isretr (f a) = ap f (issect' a).

We don't make this a typeclass instance, because we want to control when we are applying it.
An involution is an endomap that is its own inverse.
Definition isequiv_involution {X : Type} (f : X X) (isinvol : Sect f f)
: IsEquiv f
  := isequiv_adjointify f f isinvol isinvol.

Definition equiv_involution {X : Type} (f : X X) (isinvol : Sect f f)
: X <~> X
  := equiv_adjointify f f isinvol isinvol.

Several lemmas useful for rewriting.
Definition moveR_equiv_M `{IsEquiv A B f} (x : A) (y : B) (p : x = f^-1 y)
  : (f x = y)
  := ap f p @ eisretr f y.

Definition moveL_equiv_M `{IsEquiv A B f} (x : A) (y : B) (p : f^-1 y = x)
  : (y = f x)
  := (eisretr f y)^ @ ap f p.

Definition moveR_equiv_V `{IsEquiv A B f} (x : B) (y : A) (p : x = f y)
  : (f^-1 x = y)
  := ap (f^-1) p @ eissect f y.

Definition moveL_equiv_V `{IsEquiv A B f} (x : B) (y : A) (p : f y = x)
  : (y = f^-1 x)
  := (eissect f y)^ @ ap (f^-1) p.

Equivalence preserves contractibility (which of course is trivial under univalence).
Lemma contr_equiv A {B} (f : A B) `{IsEquiv A B f} `{Contr A}
  : Contr B.

Definition contr_equiv' A {B} `(f : A <~> B) `{Contr A}
  : Contr B
  := contr_equiv A f.

Any two contractible types are equivalent.
Global Instance isequiv_contr_contr {A B : Type}
       `{Contr A} `{Contr B} (f : A B)
  : IsEquiv f
  := BuildIsEquiv _ _ f (fun _ ⇒ (center A))
                  (fun xpath_contr _ _)
                  (fun xpath_contr _ _)
                  (fun xpath_contr _ _).

Lemma equiv_contr_contr {A B : Type} `{Contr A} `{Contr B}
  : (A <~> B).

Assuming function extensionality, composing with an equivalence is itself an equivalence

Global Instance isequiv_precompose `{Funext} {A B C : Type}
  (f : A B) `{IsEquiv A B f}
  : IsEquiv (fun (g:BC) ⇒ g o f) | 1000
  := isequiv_adjointify (fun (g:BC) ⇒ g o f)
    (fun hh o f^-1)
    (fun hpath_forall _ _ (fun xap h (eissect f x)))
    (fun gpath_forall _ _ (fun yap g (eisretr f y))).

Definition equiv_precompose `{Funext} {A B C : Type}
  (f : A B) `{IsEquiv A B f}
  : (B C) <~> (A C)
  := BuildEquiv _ _ (fun (g:BC) ⇒ g o f) _.

Definition equiv_precompose' `{Funext} {A B C : Type} (f : A <~> B)
  : (B C) <~> (A C)
  := BuildEquiv _ _ (fun (g:BC) ⇒ g o f) _.

Global Instance isequiv_postcompose `{Funext} {A B C : Type}
  (f : B C) `{IsEquiv B C f}
  : IsEquiv (fun (g:AB) ⇒ f o g) | 1000
  := isequiv_adjointify (fun (g:AB) ⇒ f o g)
    (fun hf^-1 o h)
    (fun hpath_forall _ _ (fun xeisretr f (h x)))
    (fun gpath_forall _ _ (fun yeissect f (g y))).

Definition equiv_postcompose `{Funext} {A B C : Type}
  (f : B C) `{IsEquiv B C f}
  : (A B) <~> (A C)
  := BuildEquiv _ _ (fun (g:AB) ⇒ f o g) _.

Definition equiv_postcompose' `{Funext} {A B C : Type} (f : B <~> C)
  : (A B) <~> (A C)
  := BuildEquiv _ _ (fun (g:AB) ⇒ f o g) _.

Conversely, if pre- or post-composing with a function is always an equivalence, then that function is also an equivalence. It's convenient to know that we only need to assume the equivalence when the other type is the domain or the codomain.

Definition isequiv_isequiv_precompose {A B : Type} (f : A B)
  (precomp := (fun (C : Type) (h : B C) ⇒ h o f))
  (Aeq : IsEquiv (precomp A)) (Beq : IsEquiv (precomp B))
  : IsEquiv f.


If f is an equivalence, then so is ap f. We are lazy and use adjointify.
Global Instance isequiv_ap `{IsEquiv A B f} (x y : A)
  : IsEquiv (@ap A B f x y) | 1000
  := isequiv_adjointify (ap f)
  (fun q(eissect f x)^ @ ap f^-1 q @ eissect f y)
  (fun q
    ap_pp f _ _
    @ whiskerR (ap_pp f _ _) _
    @ ((ap_V f _ @ inverse2 (eisadj f _)^)
      @@ (ap_compose f^-1 f _)^
      @@ (eisadj f _)^)
    @ concat_pA1_p (eisretr f) _ _
    @ whiskerR (concat_Vp _) _
    @ concat_1p _)
  (fun p
    whiskerR (whiskerL _ (ap_compose f f^-1 _)^) _
    @ concat_pA1_p (eissect f) _ _
    @ whiskerR (concat_Vp _) _
    @ concat_1p _).

The function equiv_ind says that given an equivalence f : A <~> B, and a hypothesis from B, one may always assume that the hypothesis is in the image of e.
In fibrational terms, if we have a fibration over B which has a section once pulled back along an equivalence f : A <~> B, then it has a section over all of B.

Definition equiv_ind `{IsEquiv A B f} (P : B Type)
  : ( x:A, P (f x)) y:B, P y
  := fun g ytransport P (eisretr f y) (g (f^-1 y)).


Definition equiv_ind_comp `{IsEquiv A B f} (P : B Type)
  (df : x:A, P (f x)) (x : A)
  : equiv_ind f P df (f x) = df x.

Using equiv_ind, we define a handy little tactic which introduces a variable and simultaneously substitutes it along an equivalence.


equiv_composeR', a flipped version of equiv_compose', is (like concatR) most often useful partially applied, to give the “first half” of an equivalence one is constructing and leave the rest as a subgoal. One could similarly define equiv_composeR as a flip of equiv_compose, but it doesn’t seem so useful since it doesn’t leave the remaining equivalence as a subgoal.
Definition equiv_composeR' {A B C} (f : A <~> B) (g : B <~> C)
  := equiv_compose' g f.


It's often convenient when constructing a chain of equivalences to use equiv_compose', etc. But when we treat an Equiv object constructed in that way as a function, via the coercion equiv_fun, Coq sometimes needs a little help to realize that the result is the same as ordinary composition. This tactic provides that help.


Definition transport_paths_l {A : Type} {x1 x2 y : A} (p : x1 = x2) (q : x1 = y)
  : transport (fun xx = y) p q = p^ @ q.

Definition transport_paths_r {A : Type} {x y1 y2 : A} (p : y1 = y2) (q : x = y1)
  : transport (fun yx = y) p q = q @ p.

Definition transport_paths_lr {A : Type} {x1 x2 : A} (p : x1 = x2) (q : x1 = x1)
  : transport (fun xx = x) p q = p^ @ q @ p.

Definition transport_paths_Fl {A B : Type} {f : A B} {x1 x2 : A} {y : B}
  (p : x1 = x2) (q : f x1 = y)
  : transport (fun xf x = y) p q = (ap f p)^ @ q.

Definition transport_paths_Fr {A B : Type} {g : A B} {y1 y2 : A} {x : B}
  (p : y1 = y2) (q : x = g y1)
  : transport (fun yx = g y) p q = q @ (ap g p).

Definition transport_paths_FlFr {A B : Type} {f g : A B} {x1 x2 : A}
  (p : x1 = x2) (q : f x1 = g x1)
  : transport (fun xf x = g x) p q = (ap f p)^ @ q @ (ap g p).

Definition transport_paths_FlFr_D {A : Type} {B : A Type}
  {f g : a, B a} {x1 x2 : A} (p : x1 = x2) (q : f x1 = g x1)
: transport (fun xf x = g x) p q
  = (apD f p)^ @ ap (transport B p) q @ (apD g p).

Definition transport_paths_FFlr {A B : Type} {f : A B} {g : B A} {x1 x2 : A}
  (p : x1 = x2) (q : g (f x1) = x1)
  : transport (fun xg (f x) = x) p q = (ap g (ap f p))^ @ q @ p.

Definition transport_paths_lFFr {A B : Type} {f : A B} {g : B A} {x1 x2 : A}
  (p : x1 = x2) (q : x1 = g (f x1))
  : transport (fun xx = g (f x)) p q = p^ @ q @ (ap g (ap f p)).

Definition transport_paths2 {A : Type} {x y : A}
           (p : x = y) (q : idpath x = idpath x)
: transport (fun aidpath a = idpath a) p q
  = (concat_Vp p)^
    @ whiskerL p^ ((concat_1p p)^ @ whiskerR q p @ concat_1p p)
    @ concat_Vp p.

Definition equiv_ap `(f : A B) `{IsEquiv A B f} (x y : A)
  : (x = y) <~> (f x = f y)
  := BuildEquiv _ _ (ap f) _.


Definition equiv_ap' `(f : A <~> B) (x y : A)
  : (x = y) <~> (f x = f y)
  := equiv_ap f x y.

Definition equiv_inj `(f : A B) `{IsEquiv A B f} {x y : A}
  : (f x = f y) (x = y)
  := (ap f)^-1.

Path operations are equivalences


Global Instance isequiv_path_inverse {A : Type} (x y : A)
  : IsEquiv (@inverse A x y) | 0.

Definition equiv_path_inverse {A : Type} (x y : A)
  : (x = y) <~> (y = x)
  := BuildEquiv _ _ (@inverse A x y) _.

Global Instance isequiv_concat_l {A : Type} `(p : x = y:>A) (z : A)
  : IsEquiv (@transitivity A _ _ x y z p) | 0.

Definition equiv_concat_l {A : Type} `(p : x = y) (z : A)
  : (y = z) <~> (x = z)
  := BuildEquiv _ _ (concat p) _.

Global Instance isequiv_concat_r {A : Type} `(p : y = z) (x : A)
  : IsEquiv (fun q:x=yq @ p) | 0.

Definition equiv_concat_r {A : Type} `(p : y = z) (x : A)
  : (x = y) <~> (x = z)
  := BuildEquiv _ _ (fun qq @ p) _.

Global Instance isequiv_concat_lr {A : Type} {x x' y y' : A} (p : x' = x) (q : y = y')
  : IsEquiv (fun r:x=yp @ r @ q) | 0
  := @isequiv_compose _ _ (fun rp @ r) _ _ (fun rr @ q) _.

Definition equiv_concat_lr {A : Type} {x x' y y' : A} (p : x' = x) (q : y = y')
  : (x = y) <~> (x' = y')
  := BuildEquiv _ _ (fun r:x=yp @ r @ q) _.

Global Instance isequiv_whiskerL {A} {x y z : A} (p : x = y) {q r : y = z}
: IsEquiv (@whiskerL A x y z p q r).

Definition equiv_whiskerL {A} {x y z : A} (p : x = y) (q r : y = z)
: (q = r) <~> (p @ q = p @ r)
  := BuildEquiv _ _ (whiskerL p) _.

Definition equiv_cancelL {A} {x y z : A} (p : x = y) (q r : y = z)
: (p @ q = p @ r) <~> (q = r)
  := equiv_inverse (equiv_whiskerL p q r).

Definition isequiv_cancelL {A} {x y z : A} (p : x = y) (q r : y = z)
  : IsEquiv (cancelL p q r).

Global Instance isequiv_whiskerR {A} {x y z : A} {p q : x = y} (r : y = z)
: IsEquiv (fun h ⇒ @whiskerR A x y z p q h r).

Definition equiv_whiskerR {A} {x y z : A} (p q : x = y) (r : y = z)
: (p = q) <~> (p @ r = q @ r)
  := BuildEquiv _ _ (fun hwhiskerR h r) _.

Definition equiv_cancelR {A} {x y z : A} (p q : x = y) (r : y = z)
: (p @ r = q @ r) <~> (p = q)
  := equiv_inverse (equiv_whiskerR p q r).

Definition isequiv_cancelR {A} {x y z : A} (p q : x = y) (r : y = z)
  : IsEquiv (cancelR p q r).

We can use these to build up more complicated equivalences.
In particular, all of the move family are equivalences.
(Note: currently, some but not all of these isequiv_ lemmas have corresponding equiv_ lemmas. Also, they do *not* currently contain the computational content that e.g. the inverse of moveR_Mp is moveL_Vp; perhaps it would be useful if they did?

Global Instance isequiv_moveR_Mp
 {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : y = x)
: IsEquiv (moveR_Mp p q r).

Definition equiv_moveR_Mp
  {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : y = x)
: (p = r^ @ q) <~> (r @ p = q)
:= BuildEquiv _ _ (moveR_Mp p q r) _.

Global Instance isequiv_moveR_pM
  {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : y = x)
: IsEquiv (moveR_pM p q r).

Definition equiv_moveR_pM
  {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : y = x)
: (r = q @ p^) <~> (r @ p = q)
:= BuildEquiv _ _ (moveR_pM p q r) _.

Global Instance isequiv_moveR_Vp
  {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : x = y)
: IsEquiv (moveR_Vp p q r).

Definition equiv_moveR_Vp
  {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : x = y)
: (p = r @ q) <~> (r^ @ p = q)
:= BuildEquiv _ _ (moveR_Vp p q r) _.

Global Instance isequiv_moveR_pV
  {A : Type} {x y z : A} (p : z = x) (q : y = z) (r : y = x)
: IsEquiv (moveR_pV p q r).

Definition equiv_moveR_pV
  {A : Type} {x y z : A} (p : z = x) (q : y = z) (r : y = x)
: (r = q @ p) <~> (r @ p^ = q)
:= BuildEquiv _ _ (moveR_pV p q r) _.

Global Instance isequiv_moveL_Mp
  {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : y = x)
: IsEquiv (moveL_Mp p q r).

Definition equiv_moveL_Mp
  {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : y = x)
: (r^ @ q = p) <~> (q = r @ p)
:= BuildEquiv _ _ (moveL_Mp p q r) _.

Definition isequiv_moveL_pM
  {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : y = x)
: IsEquiv (moveL_pM p q r).

Definition equiv_moveL_pM
  {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : y = x) :
  q @ p^ = r <~> q = r @ p
  := BuildEquiv _ _ _ (isequiv_moveL_pM p q r).

Global Instance isequiv_moveL_Vp
  {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : x = y)
: IsEquiv (moveL_Vp p q r).

Definition equiv_moveL_Vp
  {A : Type} {x y z : A} (p : x = z) (q : y = z) (r : x = y)
: r @ q = p <~> q = r^ @ p
:= BuildEquiv _ _ (moveL_Vp p q r) _.

Global Instance isequiv_moveL_pV
  {A : Type} {x y z : A} (p : z = x) (q : y = z) (r : y = x)
: IsEquiv (moveL_pV p q r).

Definition equiv_moveL_pV
  {A : Type} {x y z : A} (p : z = x) (q : y = z) (r : y = x)
: q @ p = r <~> q = r @ p^
:= BuildEquiv _ _ (moveL_pV p q r) _.

Definition isequiv_moveL_1M {A : Type} {x y : A} (p q : x = y)
: IsEquiv (moveL_1M p q).

Definition isequiv_moveL_M1 {A : Type} {x y : A} (p q : x = y)
: IsEquiv (moveL_M1 p q).

Definition isequiv_moveL_1V {A : Type} {x y : A} (p : x = y) (q : y = x)
: IsEquiv (moveL_1V p q).

Definition isequiv_moveL_V1 {A : Type} {x y : A} (p : x = y) (q : y = x)
: IsEquiv (moveL_V1 p q).

Definition isequiv_moveR_M1 {A : Type} {x y : A} (p q : x = y)
: IsEquiv (moveR_M1 p q).

Definition isequiv_moveR_1M {A : Type} {x y : A} (p q : x = y)
: IsEquiv (moveR_1M p q).

Definition isequiv_moveR_1V {A : Type} {x y : A} (p : x = y) (q : y = x)
: IsEquiv (moveR_1V p q).

Definition isequiv_moveR_V1 {A : Type} {x y : A} (p : x = y) (q : y = x)
: IsEquiv (moveR_V1 p q).

Definition moveR_moveL_transport_V {A : Type} (P : A Type) {x y : A}
           (p : x = y) (u : P x) (v : P y) (q : transport P p u = v)
  : moveR_transport_p P p u v (moveL_transport_V P p u v q) = q.

Definition moveL_moveR_transport_p {A : Type} (P : A Type) {x y : A}
           (p : x = y) (u : P x) (v : P y) (q : u = transport P p^ v)
  : moveL_transport_V P p u v (moveR_transport_p P p u v q) = q.

Global Instance isequiv_moveR_transport_p {A : Type} (P : A Type) {x y : A}
  (p : x = y) (u : P x) (v : P y)
: IsEquiv (moveR_transport_p P p u v).

Definition equiv_moveR_transport_p {A : Type} (P : A Type) {x y : A}
  (p : x = y) (u : P x) (v : P y)
: u = transport P p^ v <~> transport P p u = v
:= BuildEquiv _ _ (moveR_transport_p P p u v) _.

Definition moveR_moveL_transport_p {A : Type} (P : A Type) {x y : A}
           (p : y = x) (u : P x) (v : P y) (q : transport P p^ u = v)
  : moveR_transport_V P p u v (moveL_transport_p P p u v q) = q.

Definition moveL_moveR_transport_V {A : Type} (P : A Type) {x y : A}
           (p : y = x) (u : P x) (v : P y) (q : u = transport P p v)
  : moveL_transport_p P p u v (moveR_transport_V P p u v q) = q.

Global Instance isequiv_moveR_transport_V {A : Type} (P : A Type) {x y : A}
  (p : y = x) (u : P x) (v : P y)
: IsEquiv (moveR_transport_V P p u v).

Definition equiv_moveR_transport_V {A : Type} (P : A Type) {x y : A}
  (p : y = x) (u : P x) (v : P y)
: u = transport P p v <~> transport P p^ u = v
:= BuildEquiv _ _ (moveR_transport_V P p u v) _.

Global Instance isequiv_moveL_transport_V {A : Type} (P : A Type) {x y : A}
  (p : x = y) (u : P x) (v : P y)
: IsEquiv (moveL_transport_V P p u v).

Definition equiv_moveL_transport_V {A : Type} (P : A Type) {x y : A}
  (p : x = y) (u : P x) (v : P y)
: transport P p u = v <~> u = transport P p^ v
:= BuildEquiv _ _ (moveL_transport_V P p u v) _.

Global Instance isequiv_moveL_transport_p {A : Type} (P : A Type) {x y : A}
  (p : y = x) (u : P x) (v : P y)
: IsEquiv (moveL_transport_p P p u v).

Definition equiv_moveL_transport_p {A : Type} (P : A Type) {x y : A}
  (p : y = x) (u : P x) (v : P y)
: transport P p^ u = v <~> u = transport P p v
:= BuildEquiv _ _ (moveL_transport_p P p u v) _.

Global Instance isequiv_moveR_equiv_M `{IsEquiv A B f} (x : A) (y : B)
: IsEquiv (@moveR_equiv_M A B f _ x y).

Definition equiv_moveR_equiv_M `{IsEquiv A B f} (x : A) (y : B)
  : (x = f^-1 y) <~> (f x = y)
  := BuildEquiv _ _ (@moveR_equiv_M A B f _ x y) _.

Global Instance isequiv_moveR_equiv_V `{IsEquiv A B f} (x : B) (y : A)
: IsEquiv (@moveR_equiv_V A B f _ x y).

Definition equiv_moveR_equiv_V `{IsEquiv A B f} (x : B) (y : A)
  : (x = f y) <~> (f^-1 x = y)
  := BuildEquiv _ _ (@moveR_equiv_V A B f _ x y) _.

Global Instance isequiv_moveL_equiv_M `{IsEquiv A B f} (x : A) (y : B)
: IsEquiv (@moveL_equiv_M A B f _ x y).

Definition equiv_moveL_equiv_M `{IsEquiv A B f} (x : A) (y : B)
  : (f^-1 y = x) <~> (y = f x)
  := BuildEquiv _ _ (@moveL_equiv_M A B f _ x y) _.

Global Instance isequiv_moveL_equiv_V `{IsEquiv A B f} (x : B) (y : A)
: IsEquiv (@moveL_equiv_V A B f _ x y).

Definition equiv_moveL_equiv_V `{IsEquiv A B f} (x : B) (y : A)
  : (f y = x) <~> (y = f^-1 x)
  := BuildEquiv _ _ (@moveL_equiv_V A B f _ x y) _.

Dependent paths

Usually, a dependent path over p:x1=x2 in P:AType between y1:P x1 and y2:P x2 is a path transport P p y1 = y2 in P x2. However, when P is a path space, these dependent paths have a more convenient description: rather than transporting the left side both forwards and backwards, we transport both sides of the equation forwards, forming a sort of "naturality square".
We use the same naming scheme as for the transport lemmas.

Definition dpath_path_l {A : Type} {x1 x2 y : A}
  (p : x1 = x2) (q : x1 = y) (r : x2 = y)
  : q = p @ r
  <~>
  transport (fun xx = y) p q = r.

Definition dpath_path_r {A : Type} {x y1 y2 : A}
  (p : y1 = y2) (q : x = y1) (r : x = y2)
  : q @ p = r
  <~>
  transport (fun yx = y) p q = r.

Definition dpath_path_lr {A : Type} {x1 x2 : A}
  (p : x1 = x2) (q : x1 = x1) (r : x2 = x2)
  : q @ p = p @ r
  <~>
  transport (fun xx = x) p q = r.

Definition dpath_path_Fl {A B : Type} {f : A B} {x1 x2 : A} {y : B}
  (p : x1 = x2) (q : f x1 = y) (r : f x2 = y)
  : q = ap f p @ r
  <~>
  transport (fun xf x = y) p q = r.

Definition dpath_path_Fr {A B : Type} {g : A B} {x : B} {y1 y2 : A}
  (p : y1 = y2) (q : x = g y1) (r : x = g y2)
  : q @ ap g p = r
  <~>
  transport (fun yx = g y) p q = r.

Definition dpath_path_FlFr {A B : Type} {f g : A B} {x1 x2 : A}
  (p : x1 = x2) (q : f x1 = g x1) (r : f x2 = g x2)
  : q @ ap g p = ap f p @ r
  <~>
  transport (fun xf x = g x) p q = r.

Definition dpath_path_FFlr {A B : Type} {f : A B} {g : B A}
  {x1 x2 : A} (p : x1 = x2) (q : g (f x1) = x1) (r : g (f x2) = x2)
  : q @ p = ap g (ap f p) @ r
  <~>
  transport (fun xg (f x) = x) p q = r.

Definition dpath_path_lFFr {A B : Type} {f : A B} {g : B A}
  {x1 x2 : A} (p : x1 = x2) (q : x1 = g (f x1)) (r : x2 = g (f x2))
  : q @ ap g (ap f p) = p @ r
  <~>
  transport (fun xx = g (f x)) p q = r.

Definition dpath_paths2 {A : Type} {x y : A}
           (p : x = y) (q : idpath x = idpath x)
           (r : idpath y = idpath y)
: (concat_1p p)^ @ whiskerR q p @ concat_1p p
  = (concat_p1 p)^ @ whiskerL p r @ concat_p1 p
  <~>
  transport (fun aidpath a = idpath a) p q = r.

Universal mapping property


Global Instance isequiv_paths_ind `{Funext} {A : Type} (a : A)
  (P : x, (a = x) Type)
  : IsEquiv (paths_ind a P) | 0.

Definition equiv_paths_ind `{Funext} {A : Type} (a : A)
  (P : x, (a = x) Type)
  : P a 1 <~> x p, P x p
  := BuildEquiv _ _ (paths_ind a P) _.


Section AssumeFunext.
Context `{Funext}.

Paths

Paths p : f = g in a function type x:X, P x are equivalent to functions taking values in path types, H : x:X, f x = g x, or concisely, H : f == g.
This equivalence, however, is just the combination of apD10 and function extensionality funext, and as such, path_forall, et seq. are given in the Overture:
Now we show how these things compute.

Definition apD10_path_forall `{P : A Type}
  (f g : x, P x) (h : f == g)
  : apD10 (path_forall _ _ h) == h
  := apD10 (eisretr apD10 h).

Definition eta_path_forall `{P : A Type}
  (f g : x, P x) (p : f = g)
  : path_forall _ _ (apD10 p) = p
  := eissect apD10 p.

Definition path_forall_1 `{P : A Type} (f : x, P x)
  : (path_forall f f (fun x ⇒ 1)) = 1
  := eta_path_forall f f 1.

The identification of the path space of a dependent function space, up to equivalence, is of course just funext.

Definition equiv_apD10 `{Funext} {A : Type} (P : A Type) f g
: (f = g) <~> (f == g)
  := BuildEquiv _ _ (@apD10 A P f g) _.

Global Instance isequiv_path_forall `{P : A Type} (f g : x, P x)
  : IsEquiv (path_forall f g) | 0
  := @isequiv_inverse _ _ (@apD10 A P f g) _.

Definition equiv_path_forall `{P : A Type} (f g : x, P x)
  : (f == g) <~> (f = g)
  := BuildEquiv _ _ (path_forall f g) _.


Path algebra


Definition path_forall_pp `{P : A Type} (f g h : x, P x)
           (p : f == g) (q : g == h)
: path_forall f h (fun xp x @ q x) = path_forall f g p @ path_forall g h q.

Definition path_forall_V `{P : A Type} (f g : x, P x)
           (p : f == g)
  : path_forall _ _ (fun x(p x)^) = (path_forall _ _ p)^.

Transport

The concrete description of transport in sigmas and pis is rather trickier than in the other types. In particular, these cannot be described just in terms of transport in simpler types; they require the full Id-elim rule by way of "dependent transport" transportD.
In particular this indicates why "transport" alone cannot be fully defined by induction on the structure of types, although Id-elim/transportD can be (cf. Observational Type Theory). A more thorough set of lemmas, along the lines of the present ones but dealing with Id-elim rather than just transport, might be nice to have eventually?
Definition transport_forall
  {A : Type} {P : A Type} {C : x, P x Type}
  {x1 x2 : A} (p : x1 = x2) (f : y : P x1, C x1 y)
  : (transport (fun x y : P x, C x y) p f)
    == (fun y
       transport (C x2) (transport_pV _ _ _) (transportD _ _ p _ (f (p^ # y)))).
Defined.

A special case of transport_forall where the type P does not depend on A, and so it is just a fixed type B.
Definition transport_forall_constant
  {A B : Type} {C : A B Type}
  {x1 x2 : A} (p : x1 = x2) (f : y : B, C x1 y)
  : (transport (fun x y : B, C x y) p f)
    == (fun ytransport (fun xC x y) p (f y)).
Defined.

Definition apD_transport_forall_constant
  {A B : Type} (C : A B Type)
  {x1 x2 : A} (p : x1 = x2) (f : y : B, C x1 y)
  {y1 y2 : B} (q : y1 = y2)
: apD (transport (fun x y : B, C x y) p f) q
  = ap (transport (C x2) q) (transport_forall_constant p f y1)
    @ transport_transport C p q (f y1)
    @ ap (transport (fun x : AC x y2) p) (apD f q)
    @ (transport_forall_constant p f y2)^.

Maps on paths

The action of maps given by application.
Definition ap_apply_lD {A} {B : A Type} {f g : x, B x} (p : f = g) (z : A)
  : ap (fun ff z) p = apD10 p z
:= 1.

Definition ap_apply_lD2 {A} {B : A Type} { C : x, B x Type}
           {f g : x y, C x y} (p : f = g) (z1 : A) (z2 : B z1)
  : ap (fun ff z1 z2) p = apD10 (apD10 p z1) z2.

The action of maps given by lambda.
Definition ap_lambdaD {A B : Type} {C : B Type} {x y : A} (p : x = y) (M : a b, C b) :
  ap (fun a bM a b) p =
  path_forall _ _ (fun bap (fun aM a b) p).

Dependent paths

Usually, a dependent path over p:x1=x2 in P:AType between y1:P x1 and y2:P x2 is a path transport P p y1 = y2 in P x2. However, when P is a function space, these dependent paths have a more convenient description: rather than transporting the argument of y1 forwards and backwards, we transport only forwards but on both sides of the equation, yielding a "naturality square".

Definition dpath_forall
  {A:Type} (B:A Type) (C: a, B a Type) (x1 x2:A) (p:x1=x2)
  (f: y1:B x1, C x1 y1) (g: (y2:B x2), C x2 y2)
  : ( (y1:B x1), transportD B C p y1 (f y1) = g (transport B p y1))
  <~>
  (transport (fun x y:B x, C x y) p f = g).

Definition dpath_forall_constant
  {A B:Type} (C : A B Type) (x1 x2:A) (p:x1=x2)
  (f: (y1:B), C x1 y1) (g: (y2:B), C x2 y2)
  : ( (y1:B), transport (fun xC x y1) p (f y1) = g y1)
  <~>
  (transport (fun x y:B, C x y) p f = g).

Functorial action

The functoriality of is slightly subtle: it is contravariant in the domain type and covariant in the codomain, but the codomain is dependent on the domain.
Definition functor_forall `{P : A Type} `{Q : B Type}
    (f0 : B A) (f1 : b:B, P (f0 b) Q b)
  : ( a:A, P a) ( b:B, Q b)
  := (fun g bf1 _ (g (f0 b))).

Definition ap_functor_forall `{P : A Type} `{Q : B Type}
    (f0 : B A) (f1 : b:B, P (f0 b) Q b)
    (g g' : a:A, P a) (h : g == g')
  : ap (functor_forall f0 f1) (path_forall _ _ h)
    = path_forall _ _ (fun b:B ⇒ (ap (f1 b) (h (f0 b)))).

Definition functor_forall_compose
           `{P : A Type} `{Q : B Type} `{R : C Type}
           (f0 : B A) (f1 : b:B, P (f0 b) Q b)
           (g0 : C B) (g1 : c:C, Q (g0 c) R c)
           (k : a, P a)
  : functor_forall g0 g1 (functor_forall f0 f1 k) == functor_forall (f0 o g0) (fun cg1 c o f1 (g0 c)) k
  := fun a ⇒ 1.

Equivalences


Global Instance isequiv_functor_forall `{P : A Type} `{Q : B Type}
  `{IsEquiv B A f} `{ b, @IsEquiv (P (f b)) (Q b) (g b)}
  : IsEquiv (functor_forall f g) | 1000.

Definition equiv_functor_forall `{P : A Type} `{Q : B Type}
  (f : B A) `{IsEquiv B A f}
  (g : b, P (f b) Q b)
  `{ b, @IsEquiv (P (f b)) (Q b) (g b)}
  : ( a, P a) <~> ( b, Q b)
  := BuildEquiv _ _ (functor_forall f g) _.

Definition equiv_functor_forall' `{P : A Type} `{Q : B Type}
  (f : B <~> A) (g : b, P (f b) <~> Q b)
  : ( a, P a) <~> ( b, Q b)
  := equiv_functor_forall f g.

Definition equiv_functor_forall_id `{P : A Type} `{Q : A Type}
  (g : a, P a <~> Q a)
  : ( a, P a) <~> ( a, Q a)
  := equiv_functor_forall (equiv_idmap A) g.

Definition equiv_functor_forall_pb {A B : Type} {P : A Type}
  (f : B <~> A)
  : ( a, P a) <~> ( b, P (f b))
  := equiv_functor_forall' (Q := P o f) f (fun bequiv_idmap).

Definition equiv_functor_forall_pf {A B : Type} {Q : B Type}
  (f : B <~> A)
  : ( a, (Q (f^-1 a))) <~> ( b, Q b).

There is another way to make forall functorial that acts on on equivalences only.

Definition equiv_functor_forall_covariant
           `{P : A Type} `{Q : B Type}
           (f : A <~> B) (g : a, P a <~> Q (f a))
  : ( a, P a) <~> ( b, Q b).

Definition equiv_functor_forall_covariant_compose
           `{P : A Type} `{Q : B Type} `{R : C Type}
           (f0 : A <~> B) (f1 : a, P a <~> Q (f0 a))
           (g0 : B <~> C) (g1 : b, Q b <~> R (g0 b))
           (h : a, P a) (c : C)
  : equiv_functor_forall_covariant g0 g1 (equiv_functor_forall_covariant f0 f1 h) c
    = equiv_functor_forall_covariant (g0 oE f0) (fun ag1 (f0 a) oE f1 a) h c.

Truncatedness: any dependent product of n-types is an n-type


Global Instance contr_forall `{P : A Type} `{ a, Contr (P a)}
  : Contr ( a, P a) | 100.


Contractibility: A product over a contractible type is equivalent to the fiber over the center.


Definition equiv_contr_forall `{Contr A} `(P : A Type)
: ( a, P a) <~> P (center A).

Symmetry of curried arguments

Using the standard Haskell name for this, as it’s a handy utility function.
Note: not sure if P will usually be deducible, or whether it would be better explicit.
Definition flip `{P : A B Type}
  : ( a b, P a b) ( b a, P a b)
  := fun f b af a b.

Global Instance isequiv_flip `{P : A B Type}
  : IsEquiv (@flip _ _ P) | 0.

Definition equiv_flip `(P : A B Type)
  : ( a b, P a b) <~> ( b a, P a b)
  := BuildEquiv _ _ (@flip _ _ P) _.

End AssumeFunext.


In homotopy type theory, We think of elements of Type as spaces, homotopy types, or weak omega-groupoids. A type family P : A Type corresponds to a fibration whose base is A and whose fiber over x is P x.
From such a P we can build a total space over the base space A so that the fiber over x : A is P x. This is just Coq's dependent sum construction, written as sigT P or {x : A & P x}. The elements of {x : A & P x} are pairs, written existT P x y in Coq, where x : A and y : P x. In Common.v we defined the notation (x;y) to mean existT _ x y.
The base and fiber components of a point in the total space are extracted with the two projections pr1 and pr2.

Unpacking

Sometimes we would like to prove Q u where u : {x : A & P x} by writing u as a pair (pr1 u ; pr2 u). This is accomplished by sigT_unpack. We want tight control over the proof, so we just write it down even though is looks a bit scary.

Definition unpack_sigma `{P : A Type} (Q : sigT P Type) (u : sigT P)
: Q (u.1; u.2) Q u
  := idmap.


Eta conversion


Definition eta_sigma `{P : A Type} (u : sigT P)
  : (u.1; u.2) = u
  := 1.


Definition eta2_sigma `{P : (a : A) (b : B a), Type}
           (u : sigT (fun asigT (P a)))
  : (u.1; (u.2.1; u.2.2)) = u
  := 1.


Definition eta3_sigma `{P : (a : A) (b : B a) (c : C a b), Type}
           (u : sigT (fun asigT (fun bsigT (P a b))))
  : (u.1; (u.2.1; (u.2.2.1; u.2.2.2))) = u
  := 1.


Paths

A path in a total space is commonly shown component wise. Because we use this over and over, we write down the proofs by hand to make sure they are what we think they should be.
With this version of the function, we often have to give u and v explicitly, so we make them explicit arguments.
Definition path_sigma_uncurried {A : Type} (P : A Type) (u v : sigT P)
           (pq : {p : u.1 = v.1 & p # u.2 = v.2})
: u = v.
Defined.

This is the curried one you usually want to use in practice. We define it in terms of the uncurried one, since it's the uncurried one that is proven below to be an equivalence.
Definition path_sigma {A : Type} (P : A Type) (u v : sigT P)
           (p : u.1 = v.1) (q : p # u.2 = v.2)
: u = v
  := path_sigma_uncurried P u v (p;q).

A contravariant instance of path_sigma_uncurried
Definition path_sigma_uncurried_contra {A : Type} (P : A Type) (u v : sigT P)
           (pq : {p : u.1 = v.1 & u.2 = p^ # v.2})
: u = v
  := (path_sigma_uncurried P v u (pq.1^;pq.2^))^.

A variant of Forall.dpath_forall from which uses dependent sums to package things. It cannot go into Forall because Sigma depends on Forall.

Definition dpath_forall'
           {A : Type } (P : A Type) (Q: sigT P Type) {x y : A} (h : x = y)
           (f : p, Q (x ; p)) (g : p, Q (y ; p))
:
  ( p, transport Q (path_sigma P (x ; p) (y; _) h 1) (f p) = g (h # p))
    <~>
    ( p, transportD P (fun xfun pQ ( x ; p)) h p (f p) = g (transport P h p)).

This version produces only paths between pairs, as opposed to paths between arbitrary inhabitants of dependent sum types. But it has the advantage that the components of those pairs can more often be inferred, so we make them implicit arguments.
Definition path_sigma' {A : Type} (P : A Type) {x x' : A} {y : P x} {y' : P x'}
           (p : x = x') (q : p # y = y')
: (x;y) = (x';y')
  := path_sigma P (x;y) (x';y') p q.

Projections of paths from a total space.

Definition pr1_path `{P : A Type} {u v : sigT P} (p : u = v)
: u.1 = v.1
  :=
    ap pr1 p.

Notation "p ..1" := (pr1_path p) (at level 3) : fibration_scope.

Definition pr2_path `{P : A Type} {u v : sigT P} (p : u = v)
: p..1 # u.2 = v.2
  := (transport_compose P pr1 p u.2)^
     @ (@apD {x:A & P x} _ pr2 _ _ p).

Notation "p ..2" := (pr2_path p) (at level 3) : fibration_scope.

Now we show how these things compute.

Definition pr1_path_sigma_uncurried `{P : A Type} {u v : sigT P}
           (pq : { p : u.1 = v.1 & p # u.2 = v.2 })
: (path_sigma_uncurried _ _ _ pq)..1 = pq.1.

Definition pr2_path_sigma_uncurried `{P : A Type} {u v : sigT P}
           (pq : { p : u.1 = v.1 & p # u.2 = v.2 })
: (path_sigma_uncurried _ _ _ pq)..2
  = ap (fun stransport P s u.2) (pr1_path_sigma_uncurried pq) @ pq.2.

Definition eta_path_sigma_uncurried `{P : A Type} {u v : sigT P}
           (p : u = v)
: path_sigma_uncurried _ _ _ (p..1; p..2) = p.

Lemma transport_pr1_path_sigma_uncurried
      `{P : A Type} {u v : sigT P}
      (pq : { p : u.1 = v.1 & transport P p u.2 = v.2 })
      Q
: transport (fun xQ x.1) (@path_sigma_uncurried A P u v pq)
  = transport _ pq.1.

Definition pr1_path_sigma `{P : A Type} {u v : sigT P}
           (p : u.1 = v.1) (q : p # u.2 = v.2)
: (path_sigma _ _ _ p q)..1 = p
  := pr1_path_sigma_uncurried (p; q).

Definition ap_pr1_path_sigma {A:Type} {P : A Type} {u v : sigT P}
           (p : u.1 = v.1) (q : p # u.2 = v.2)
  : ap pr1 (path_sigma _ _ _ p q) = p
  := pr1_path_sigma p q.

Definition pr2_path_sigma `{P : A Type} {u v : sigT P}
           (p : u.1 = v.1) (q : p # u.2 = v.2)
: (path_sigma _ _ _ p q)..2
  = ap (fun stransport P s u.2) (pr1_path_sigma p q) @ q
  := pr2_path_sigma_uncurried (p; q).

Definition eta_path_sigma `{P : A Type} {u v : sigT P} (p : u = v)
: path_sigma _ _ _ (p..1) (p..2) = p
  := eta_path_sigma_uncurried p.

Definition transport_pr1_path_sigma
           `{P : A Type} {u v : sigT P}
           (p : u.1 = v.1) (q : p # u.2 = v.2)
           Q
: transport (fun xQ x.1) (@path_sigma A P u v p q)
  = transport _ p
  := transport_pr1_path_sigma_uncurried (p; q) Q.

This lets us identify the path space of a sigma-type, up to equivalence.

Global Instance isequiv_path_sigma `{P : A Type} {u v : sigT P}
: IsEquiv (path_sigma_uncurried P u v) | 0.

Definition equiv_path_sigma `(P : A Type) (u v : sigT P)
: {p : u.1 = v.1 & p # u.2 = v.2} <~> (u = v)
  := BuildEquiv _ _ (path_sigma_uncurried P u v) _.

Instance isequiv_path_sigma_contra `{P : A Type} {u v : sigT P}
  : IsEquiv (path_sigma_uncurried_contra P u v) | 0.
Defined.

Definition equiv_path_sigma_contra {A : Type} `(P : A Type) (u v : sigT P)
  : {p : u.1 = v.1 & u.2 = p^ # v.2} <~> (u = v)
  := BuildEquiv _ _ (path_sigma_uncurried_contra P u v) _.

This identification respects path concatenation.

Definition path_sigma_pp_pp {A : Type} (P : A Type) {u v w : sigT P}
           (p1 : u.1 = v.1) (q1 : p1 # u.2 = v.2)
           (p2 : v.1 = w.1) (q2 : p2 # v.2 = w.2)
: path_sigma P u w (p1 @ p2)
             (transport_pp P p1 p2 u.2 @ ap (transport P p2) q1 @ q2)
  = path_sigma P u v p1 q1 @ path_sigma P v w p2 q2.

Definition path_sigma_pp_pp' {A : Type} (P : A Type)
           {u1 v1 w1 : A} {u2 : P u1} {v2 : P v1} {w2 : P w1}
           (p1 : u1 = v1) (q1 : p1 # u2 = v2)
           (p2 : v1 = w1) (q2 : p2 # v2 = w2)
: path_sigma' P (p1 @ p2)
              (transport_pp P p1 p2 u2 @ ap (transport P p2) q1 @ q2)
  = path_sigma' P p1 q1 @ path_sigma' P p2 q2
  := @path_sigma_pp_pp A P (u1;u2) (v1;v2) (w1;w2) p1 q1 p2 q2.

Definition path_sigma_p1_1p' {A : Type} (P : A Type)
           {u1 v1 : A} {u2 : P u1} {v2 : P v1}
           (p : u1 = v1) (q : p # u2 = v2)
: path_sigma' P p q
  = path_sigma' P p 1 @ path_sigma' P 1 q.

pr1_path also commutes with the groupoid structure.

Definition pr1_path_1 {A : Type} {P : A Type} (u : sigT P)
: (idpath u) ..1 = idpath (u .1)
  := 1.

Definition pr1_path_pp {A : Type} {P : A Type} {u v w : sigT P}
           (p : u = v) (q : v = w)
: (p @ q) ..1 = (p ..1) @ (q ..1)
  := ap_pp _ _ _.

Definition pr1_path_V {A : Type} {P : A Type} {u v : sigT P} (p : u = v)
: p^ ..1 = (p ..1)^
  := ap_V _ _.

Applying existT to one argument is the same as path_sigma with reflexivity in the first place.

Definition ap_existT {A : Type} (P : A Type) (x : A) (y1 y2 : P x)
           (q : y1 = y2)
: ap (existT P x) q = path_sigma' P 1 q.

Dependent transport is the same as transport along a path_sigma.

Definition transportD_is_transport
           {A:Type} (B:AType) (C:sigT B Type)
           (x1 x2:A) (p:x1=x2) (y:B x1) (z:C (x1;y))
: transportD B (fun a bC (a;b)) p y z
  = transport C (path_sigma' B p 1) z.

Applying a two variable function to a path_sigma.


And we can simplify when the first equality is 1.
Lemma ap_path_sigma_1p {A B : Type} {P : A Type} (F : a, P a B)
      (a : A) {x y : P a} (p : x = y)
  : ap (fun wF w.1 w.2) (path_sigma' P 1 p) = ap (fun zF a z) p.

Applying a function constructed with sigT_ind to a path_sigma can be computed. Technically this computation should probably go by way of a 2-variable ap, and should be done in the dependently typed case.



A path between paths in a total space is commonly shown component wise.
With this version of the function, we often have to give u and v explicitly, so we make them explicit arguments.
Definition path_path_sigma_uncurried {A : Type} (P : A Type) (u v : sigT P)
           (p q : u = v)
           (rs : {r : p..1 = q..1 & transport (fun xtransport P x u.2 = v.2) r p..2 = q..2})
: p = q.

This is the curried one you usually want to use in practice. We define it in terms of the uncurried one, since it's the uncurried one that is proven below to be an equivalence.
Definition path_path_sigma {A : Type} (P : A Type) (u v : sigT P)
           (p q : u = v)
           (r : p..1 = q..1)
           (s : transport (fun xtransport P x u.2 = v.2) r p..2 = q..2)
: p = q
  := path_path_sigma_uncurried P u v p q (r; s).

Transport

The concrete description of transport in sigmas (and also pis) is rather trickier than in the other types. In particular, these cannot be described just in terms of transport in simpler types; they require also the dependent transport transportD.
In particular, this indicates why "transport" alone cannot be fully defined by induction on the structure of types, although Id-elim/transportD can be (cf. Observational Type Theory). A more thorough set of lemmas, along the lines of the present ones but dealing with Id-elim rather than just transport, might be nice to have eventually?

Definition transport_sigma {A : Type} {B : A Type} {C : a:A, B a Type}
           {x1 x2 : A} (p : x1 = x2) (yz : { y : B x1 & C x1 y })
: transport (fun x{ y : B x & C x y }) p yz
  = (p # yz.1 ; transportD _ _ p yz.1 yz.2).

The special case when the second variable doesn't depend on the first is simpler.
Definition transport_sigma' {A B : Type} {C : A B Type}
           {x1 x2 : A} (p : x1 = x2) (yz : { y : B & C x1 y })
: transport (fun x{ y : B & C x y }) p yz =
  (yz.1 ; transport (fun xC x yz.1) p yz.2).

Or if the second variable contains a first component that doesn't depend on the first. Need to think about the naming of these.

Definition transport_sigma_' {A : Type} {B C : A Type}
           {D : a:A, B a C a Type}
           {x1 x2 : A} (p : x1 = x2)
           (yzw : { y : B x1 & { z : C x1 & D x1 y z } })
: transport (fun x{ y : B x & { z : C x & D x y z } }) p yzw
  = (p # yzw.1 ; (p # yzw.2.1 ; transportD2 _ _ _ p yzw.1 yzw.2.1 yzw.2.2)).

Functorial action


Definition functor_sigma `{P : A Type} `{Q : B Type}
           (f : A B) (g : a, P a Q (f a))
: sigT P sigT Q
  := fun u(f u.1 ; g u.1 u.2).

Definition ap_functor_sigma `{P : A Type} `{Q : B Type}
           (f : A B) (g : a, P a Q (f a))
           (u v : sigT P) (p : u.1 = v.1) (q : p # u.2 = v.2)
: ap (functor_sigma f g) (path_sigma P u v p q)
  = path_sigma Q (functor_sigma f g u) (functor_sigma f g v)
               (ap f p)
               ((transport_compose Q f p (g u.1 u.2))^
                @ (@ap_transport _ P (fun xQ (f x)) _ _ p g u.2)^
                @ ap (g v.1) q).

Equivalences


Global Instance isequiv_functor_sigma `{P : A Type} `{Q : B Type}
         `{IsEquiv A B f} `{ a, @IsEquiv (P a) (Q (f a)) (g a)}
: IsEquiv (functor_sigma f g) | 1000.

Definition equiv_functor_sigma `{P : A Type} `{Q : B Type}
           (f : A B) `{IsEquiv A B f}
           (g : a, P a Q (f a))
           `{ a, @IsEquiv (P a) (Q (f a)) (g a)}
: sigT P <~> sigT Q
  := BuildEquiv _ _ (functor_sigma f g) _.

Definition equiv_functor_sigma' `{P : A Type} `{Q : B Type}
           (f : A <~> B)
           (g : a, P a <~> Q (f a))
: sigT P <~> sigT Q
  := equiv_functor_sigma f g.

Definition equiv_functor_sigma_id `{P : A Type} `{Q : A Type}
           (g : a, P a <~> Q a)
: sigT P <~> sigT Q
  := equiv_functor_sigma' 1 g.

Lemma 3.11.9(i): Summing up a contractible family of types does nothing.

Global Instance isequiv_pr1_contr {A} {P : A Type}
         `{ a, Contr (P a)}
: IsEquiv (@pr1 A P) | 100.

Definition equiv_sigma_contr {A : Type} (P : A Type)
           `{ a, Contr (P a)}
: sigT P <~> A
  := BuildEquiv _ _ pr1 _.

Lemma 3.11.9(ii): Dually, summing up over a contractible type does nothing.

Definition equiv_contr_sigma {A : Type} (P : A Type) `{Contr A}
: { x : A & P x } <~> P (center A).

Associativity


Definition equiv_sigma_assoc `(P : A Type) (Q : {a : A & P a} Type)
: {a : A & {p : P a & Q (a;p)}} <~> sigT Q
  := @BuildEquiv
       _ _ _
       (@BuildIsEquiv
          {a : A & {p : P a & Q (a;p)}} (sigT Q)
          (fun apq((apq.1; apq.2.1); apq.2.2))
          (fun apq(apq.1.1; (apq.1.2; apq.2)))
          (fun _ ⇒ 1)
          (fun _ ⇒ 1)
          (fun _ ⇒ 1)).