Library UniMath.Foundations.PartD
Univalent Foundations. Vladimir Voevodsky. Feb. 2010 - Sep. 2011.
Port to coq trunk (8.4-8.5) in March 2014. The third part of the original uu0 file, created on Dec. 3, 2014.Contents
- Sections of "double fibration" (P : T -> UU) (PP : ∏ t : T, P t -> UU) and
pairs of sections
- General case
- Functions on dependent sum (to a total2)
- Functions to direct product
- Homotopy fibers of the map ∏ x : X, P x -> ∏ x : X, Q x
- The map between section spaces (dependent products) defined by the map
between the bases f : Y -> X
- General case
- Composition of functions with a weak equivalence on the left
- Sections of families over an empty type and over coproducts
- General case
- Functions from the empty type
- Functions from a coproduct
- Sections of families over contractible types and over total2 (over dependent sums)
- Theorem saying that if each member of a family is of h-level n then the
space of sections of the family is of h-level n.
- General case
- Functions to a contractible type
- Functions to a proposition
- Functions to an empty type (generalization of isapropneg)
- Theorems saying that iscontr T , isweq f etc. are of h-level 1
- Theorems saying that various pr1 maps are inclusions
- Various weak equivalences between spaces of weak equivalences
- Composition with a weak equivalence is a weak equivalence on weak equivalences
- Invertion on weak equivalences as a weak equivalence
- h-levels of spaces of weak equivalences
- Weak equivalences to and from types of h-level (S n)
- Weak equivalences to and from contractible types
- Weak equivalences to and from propositions
- Weak equivalences to and from sets
- Weak equivalences to an empty type
- Weak equivalences from an empty type
- Weak equivalences to and from unit
- Weak auto-equivalences of a type with an isolated point
Preamble
Sections of "double fibration" (P : T -> UU) (PP : ∏ t : T, P t -> UU) and pairs of sections
General case
Definition totaltoforall {X : UU} (P : X -> UU) (PP : ∏ x, P x -> UU) :
(∑ (s0 : ∏ x, P x), ∏ x, PP x (s0 x))
->
∏ x, ∑ p, PP x p.
Show proof.
Definition foralltototal {X : UU} (P : X -> UU) (PP : ∏ x, P x -> UU) :
(∏ x, ∑ p, PP x p)
->
(∑ (s0 : ∏ x, P x), ∏ x, PP x (s0 x)).
Show proof.
Theorem isweqforalltototal {X : UU} (P : X -> UU) (PP : ∏ x, P x -> UU) :
isweq (foralltototal P PP).
Show proof.
intros.
simple refine (isweq_iso (foralltototal P PP) (totaltoforall P PP) _ _).
- apply idpath.
- apply idpath.
simple refine (isweq_iso (foralltototal P PP) (totaltoforall P PP) _ _).
- apply idpath.
- apply idpath.
Theorem isweqtotaltoforall {X : UU} (P : X -> UU) (PP : ∏ x, P x -> UU) :
isweq (totaltoforall P PP).
Show proof.
intros.
simple refine (isweq_iso (totaltoforall P PP) (foralltototal P PP) _ _).
- apply idpath.
- apply idpath.
simple refine (isweq_iso (totaltoforall P PP) (foralltototal P PP) _ _).
- apply idpath.
- apply idpath.
Definition weqforalltototal {X : UU} (P : X -> UU) (PP : ∏ x, P x -> UU)
: (∏ x, ∑ y, PP x y)
≃
(∑ s : (∏ x, P x), (∏ x, PP x (s x)))
:= make_weq _ (isweqforalltototal P PP).
Definition weqtotaltoforall {X : UU} (P : X -> UU) (PP : ∏ x, P x -> UU)
: (∑ s : (∏ x, P x), (∏ x, PP x (s x)))
≃
(∏ x, ∑ y, PP x y)
:= invweq (weqforalltototal P PP).
Functions to a dependent sum (to a total2 )
Definition weqfuntototaltototal (X : UU) {Y : UU} (Q : Y -> UU)
: (X → ∑ y, Q y)
≃
(∑ f : X → Y, ∏ x, Q (f x))
:= weqforalltototal (λ x, Y) (λ x, Q).
Definition funtoprodtoprod {X Y Z : UU} (f : X -> Y × Z)
: (X -> Y) × (X -> Z)
:= make_dirprod (λ x, pr1 (f x)) (λ x, (pr2 (f x))).
Definition prodtofuntoprod {X Y Z : UU} (fg : (X -> Y) × (X -> Z))
: X -> Y × Z
:= λ x, (pr1 fg x ,, pr2 fg x).
Theorem weqfuntoprodtoprod (X Y Z : UU) :
(X -> Y × Z) ≃ (X -> Y) × (X -> Z).
Show proof.
intros.
simple refine (make_weq _ (isweq_iso (@funtoprodtoprod X Y Z)
(@prodtofuntoprod X Y Z) _ _)).
- intro a. apply funextfun. intro x. apply idpath.
- intro a. induction a as [ fy fz ]. apply idpath.
simple refine (make_weq _ (isweq_iso (@funtoprodtoprod X Y Z)
(@prodtofuntoprod X Y Z) _ _)).
- intro a. apply funextfun. intro x. apply idpath.
- intro a. induction a as [ fy fz ]. apply idpath.
Definition maponsec {X : UU} (P Q : X -> UU) (f : ∏ x, P x -> Q x) :
(∏ x, P x) -> (∏ x, Q x)
:= λ (s : ∏ x, P x) (x : X), (f x) (s x).
Definition maponsec1 {X Y : UU} (P : Y -> UU) (f : X -> Y) :
(∏ y : Y, P y) -> (∏ x, P (f x))
:= λ (sy : ∏ y : Y, P y) (x : X), sy (f x).
Definition hfibertoforall {X : UU} (P Q : X -> UU) (f : ∏ x, P x -> Q x)
(s : ∏ x, Q x) :
hfiber (maponsec _ _ f) s -> ∏ x, hfiber (f x) (s x).
Show proof.
unfold hfiber.
set (map1 := totalfun (λ (pointover : ∏ x, P x), (λ x, f x (pointover x)) = s)
(λ (pointover : ∏ x, P x), ∏ x, (f x) (pointover x) = s x)
(λ (pointover : ∏ x, P x), toforallpaths _ (λ x, f x (pointover x)) s)).
set (map2 := totaltoforall P (λ x pointover, f x pointover = s x)).
exact (map2 ∘ map1).
set (map1 := totalfun (λ (pointover : ∏ x, P x), (λ x, f x (pointover x)) = s)
(λ (pointover : ∏ x, P x), ∏ x, (f x) (pointover x) = s x)
(λ (pointover : ∏ x, P x), toforallpaths _ (λ x, f x (pointover x)) s)).
set (map2 := totaltoforall P (λ x pointover, f x pointover = s x)).
exact (map2 ∘ map1).
Definition foralltohfiber {X : UU} (P Q : X -> UU) (f : ∏ x, P x -> Q x)
(s : ∏ x, Q x) :
(∏ x, hfiber (f x) (s x)) -> hfiber (maponsec _ _ f) s.
Show proof.
unfold hfiber.
set (map2inv := foralltototal P (λ x pointover, f x pointover = s x)).
set (map1inv := totalfun (λ pointover, ∏ x, f x (pointover x) = s x)
(λ pointover, (λ x, f x (pointover x)) = s)
(λ pointover, funextsec _ (λ x, f x (pointover x)) s)).
exact (λ a, map1inv (map2inv a)).
set (map2inv := foralltototal P (λ x pointover, f x pointover = s x)).
set (map1inv := totalfun (λ pointover, ∏ x, f x (pointover x) = s x)
(λ pointover, (λ x, f x (pointover x)) = s)
(λ pointover, funextsec _ (λ x, f x (pointover x)) s)).
exact (λ a, map1inv (map2inv a)).
Theorem isweqhfibertoforall {X : UU} (P Q : X -> UU) (f : ∏ x, P x -> Q x)
(s : ∏ x, Q x) : isweq (hfibertoforall P Q f s).
Show proof.
use twooutof3c.
- exact (isweqfibtototal _ _ (λ pointover, weqtoforallpaths _ _ _)).
- apply isweqtotaltoforall.
- exact (isweqfibtototal _ _ (λ pointover, weqtoforallpaths _ _ _)).
- apply isweqtotaltoforall.
Definition weqhfibertoforall {X : UU} (P Q : X -> UU) (f : ∏ x, P x -> Q x)
(s : ∏ x, Q x)
: hfiber (maponsec P Q f) s ≃ ∏ x, hfiber (f x) (s x)
:= make_weq _ (isweqhfibertoforall P Q f s).
Theorem isweqforalltohfiber {X : UU} (P Q : X -> UU) (f : ∏ x, P x -> Q x)
(s : ∏ x, Q x) : isweq (foralltohfiber _ _ f s).
Show proof.
use (twooutof3c (Y := @total2 (forall x, P x)
(λ (s0 : forall x, P x),
forall x,
(λ x0 (pointover : P x0), f x0 pointover = s x0) x (s0 x)))).
- exact (isweqforalltototal P (λ x, (λ pointover, f x pointover = s x))).
- exact (isweqfibtototal _ _ (λ pointover, weqfunextsec _ _ _)).
(λ (s0 : forall x, P x),
forall x,
(λ x0 (pointover : P x0), f x0 pointover = s x0) x (s0 x)))).
- exact (isweqforalltototal P (λ x, (λ pointover, f x pointover = s x))).
- exact (isweqfibtototal _ _ (λ pointover, weqfunextsec _ _ _)).
Definition weqforalltohfiber {X : UU} (P Q : X -> UU) (f : ∏ x, P x -> Q x)
(s : ∏ x, Q x)
: (∏ x, hfiber (f x) (s x)) ≃ hfiber (maponsec P Q f) s
:= make_weq _ (isweqforalltohfiber P Q f s).
The weak equivalence between section spaces (dependent products) defined by a family of weak equivalences (P x) ≃ (Q x)
Corollary isweqmaponsec {X : UU} (P Q : X -> UU) (f : ∏ x, (P x) ≃ (Q x)) :
isweq (maponsec _ _ f).
Show proof.
intros. unfold isweq. intro y.
assert (is1 : iscontr (∏ x, hfiber (f x) (y x))).
{
assert (is2 : ∏ x, iscontr (hfiber (f x) (y x)))
by (intro x; apply ((pr2 (f x)) (y x))).
apply funcontr. assumption.
}
apply (iscontrweqb (weqhfibertoforall P Q f y) is1).
assert (is1 : iscontr (∏ x, hfiber (f x) (y x))).
{
assert (is2 : ∏ x, iscontr (hfiber (f x) (y x)))
by (intro x; apply ((pr2 (f x)) (y x))).
apply funcontr. assumption.
}
apply (iscontrweqb (weqhfibertoforall P Q f y) is1).
Definition weqonsecfibers {X : UU} (P Q : X -> UU) (f : ∏ x, (P x) ≃ (Q x))
: (∏ x, P x) ≃ (∏ x, Q x)
:= make_weq _ (isweqmaponsec P Q f).
Definition weqffun (X : UU) {Y Z : UU} (w : Y ≃ Z)
: (X -> Y) ≃ (X -> Z)
:= weqonsecfibers _ _ (λ x, w).
The map between section spaces (dependent products) defined by the map between the bases f : Y -> X
General case
Definition maponsec1l0 {X : UU} (P : X -> UU) (f : X -> X)
(h : ∏ x, f x = x) : (∏ x, P x) -> (∏ x, P x)
:= λ s x, transportf P (h x) (s (f x)).
Lemma maponsec1l1 {X : UU} (P : X -> UU) (x : X) (s : ∏ x, P x) :
maponsec1l0 P (λ x, x) idpath s x = s x.
Show proof.
Lemma maponsec1l2 {X : UU} (P : X -> UU) (f : X -> X) (h : ∏ x, f x = x)
(s : ∏ x, P x) x : maponsec1l0 P f h s x = s x.
Show proof.
intros.
set (map := λ (ff : (∑ (f0 : X -> X), ∏ x, (f0 x) = x)),
maponsec1l0 P (pr1 ff) (pr2 ff) s x).
assert (is1 : iscontr (∑ (f0 : X -> X), ∏ x, (f0 x) = x))
by apply funextcontr.
assert (e: (f,,h) = tpair (λ g, ∏ x, g x = x) (λ x, x) idpath)
by (apply proofirrelevancecontr; assumption).
apply (maponpaths map e).
set (map := λ (ff : (∑ (f0 : X -> X), ∏ x, (f0 x) = x)),
maponsec1l0 P (pr1 ff) (pr2 ff) s x).
assert (is1 : iscontr (∑ (f0 : X -> X), ∏ x, (f0 x) = x))
by apply funextcontr.
assert (e: (f,,h) = tpair (λ g, ∏ x, g x = x) (λ x, x) idpath)
by (apply proofirrelevancecontr; assumption).
apply (maponpaths map e).
Theorem isweqmaponsec1 {X Y : UU} (P : Y -> UU) (f : X ≃ Y) :
isweq (maponsec1 P f).
Show proof.
intros.
set (map := maponsec1 P f).
set (invf := invmap f).
set (e1 := homotweqinvweq f). set (e2 := homotinvweqweq f).
set (im1 := λ (sx : ∏ x, P (f x)) y, sx (invf y)).
set (im2 := λ (sy': ∏ y : Y, P (f (invf y))) y, transportf _ (homotweqinvweq f y) (sy' y)).
set (invmapp := λ (sx : ∏ x, P (f x)), im2 (im1 sx)).
assert (efg0 : ∏ (sx : (∏ x, P (f x))) x, (map (invmapp sx)) x = sx x).
{
intro. intro. unfold map. unfold invmapp. unfold im1. unfold im2.
unfold maponsec1. simpl. fold invf. set (ee := e2 x). fold invf in ee.
set (e3x := λ x0 : X, invmaponpathsweq f (invf (f x0)) x0
(homotweqinvweq f (f x0))).
set (e3 := e3x x).
assert (e4 : homotweqinvweq f (f x) = maponpaths f e3)
by apply (pathsinv0 (pathsweq4 f (invf (f x)) x _)).
assert (e5 : transportf P (homotweqinvweq f (f x)) (sx (invf (f x))) =
transportf P (maponpaths f e3) (sx (invf (f x))))
by apply (maponpaths (λ e40, (transportf P e40 (sx (invf (f x)))))
e4).
assert (e6 : transportf P (maponpaths f e3) (sx (invf (f x))) =
transportf (λ x, P (f x)) e3 (sx (invf (f x))))
by apply (pathsinv0 (functtransportf f P e3 (sx (invf (f x))))).
set (ff := λ x, invf (f x)).
assert (e7 : transportf (λ x, P (f x)) e3 (sx (invf (f x))) = sx x)
by apply (maponsec1l2 (λ x, P (f x)) ff e3x sx x).
apply (pathscomp0 (pathscomp0 e5 e6) e7).
}
assert (efg : ∏ sx : (∏ x, P (f x)), map (invmapp sx) = sx)
by (intro; apply (funextsec _ _ _ (efg0 sx))).
assert (egf0 : ∏ sy : (∏ y : Y, P y), ∏ y : Y, (invmapp (map sy)) y = sy y).
{
intros. unfold invmapp. unfold map. unfold im1. unfold im2.
unfold maponsec1.
set (ff := λ y : Y, f (invf y)). fold invf.
apply (maponsec1l2 P ff (homotweqinvweq f) sy y).
}
assert (egf : ∏ sy : (∏ y : Y, P y), invmapp (map sy) = sy)
by (intro; apply (funextsec _ _ _ (egf0 sy))).
apply (isweq_iso map invmapp egf efg).
set (map := maponsec1 P f).
set (invf := invmap f).
set (e1 := homotweqinvweq f). set (e2 := homotinvweqweq f).
set (im1 := λ (sx : ∏ x, P (f x)) y, sx (invf y)).
set (im2 := λ (sy': ∏ y : Y, P (f (invf y))) y, transportf _ (homotweqinvweq f y) (sy' y)).
set (invmapp := λ (sx : ∏ x, P (f x)), im2 (im1 sx)).
assert (efg0 : ∏ (sx : (∏ x, P (f x))) x, (map (invmapp sx)) x = sx x).
{
intro. intro. unfold map. unfold invmapp. unfold im1. unfold im2.
unfold maponsec1. simpl. fold invf. set (ee := e2 x). fold invf in ee.
set (e3x := λ x0 : X, invmaponpathsweq f (invf (f x0)) x0
(homotweqinvweq f (f x0))).
set (e3 := e3x x).
assert (e4 : homotweqinvweq f (f x) = maponpaths f e3)
by apply (pathsinv0 (pathsweq4 f (invf (f x)) x _)).
assert (e5 : transportf P (homotweqinvweq f (f x)) (sx (invf (f x))) =
transportf P (maponpaths f e3) (sx (invf (f x))))
by apply (maponpaths (λ e40, (transportf P e40 (sx (invf (f x)))))
e4).
assert (e6 : transportf P (maponpaths f e3) (sx (invf (f x))) =
transportf (λ x, P (f x)) e3 (sx (invf (f x))))
by apply (pathsinv0 (functtransportf f P e3 (sx (invf (f x))))).
set (ff := λ x, invf (f x)).
assert (e7 : transportf (λ x, P (f x)) e3 (sx (invf (f x))) = sx x)
by apply (maponsec1l2 (λ x, P (f x)) ff e3x sx x).
apply (pathscomp0 (pathscomp0 e5 e6) e7).
}
assert (efg : ∏ sx : (∏ x, P (f x)), map (invmapp sx) = sx)
by (intro; apply (funextsec _ _ _ (efg0 sx))).
assert (egf0 : ∏ sy : (∏ y : Y, P y), ∏ y : Y, (invmapp (map sy)) y = sy y).
{
intros. unfold invmapp. unfold map. unfold im1. unfold im2.
unfold maponsec1.
set (ff := λ y : Y, f (invf y)). fold invf.
apply (maponsec1l2 P ff (homotweqinvweq f) sy y).
}
assert (egf : ∏ sy : (∏ y : Y, P y), invmapp (map sy) = sy)
by (intro; apply (funextsec _ _ _ (egf0 sy))).
apply (isweq_iso map invmapp egf efg).
Definition weqonsecbase {X Y : UU} (P : Y -> UU) (f : X ≃ Y)
: (∏ y : Y, P y) ≃ (∏ x, P (f x))
:= make_weq _ (isweqmaponsec1 P f).
Definition iscontrsecoverempty (P : empty -> UU) : iscontr (∏ x : empty, P x).
Show proof.
Definition iscontrsecoverempty2 {X : UU} (P : X -> UU) (is : neg X) :
iscontr (∏ x, P x).
Show proof.
intros. set (w := weqtoempty is). set (w' := weqonsecbase P (invweq w)).
apply (iscontrweqb w' (iscontrsecoverempty _)).
apply (iscontrweqb w' (iscontrsecoverempty _)).
Definition secovercoprodtoprod {X Y : UU} (P : X ⨿ Y -> UU)
(a : ∏ xy : X ⨿ Y, P xy) :
(∏ x, P (ii1 x)) × (∏ y : Y, P (ii2 y))
:= make_dirprod (λ x, a (ii1 x)) (λ y : Y, a (ii2 y)).
Definition prodtosecovercoprod {X Y : UU} (P : X ⨿ Y -> UU)
(a : (∏ x, P (ii1 x)) × (∏ y : Y, P (ii2 y))) :
∏ xy : X ⨿ Y, P xy.
Show proof.
Definition weqsecovercoprodtoprod {X Y : UU} (P : X ⨿ Y -> UU) :
(∏ xy : X ⨿ Y, P xy)
≃
(∏ x, P (ii1 x)) × (∏ y : Y, P (ii2 y)).
Show proof.
intros.
use (weq_iso (secovercoprodtoprod P) (prodtosecovercoprod P)).
- intro. apply funextsec. intro t. induction t; reflexivity.
- intro a. apply pathsdirprod.
+ apply funextsec. apply homotrefl.
+ apply funextsec. apply homotrefl.
use (weq_iso (secovercoprodtoprod P) (prodtosecovercoprod P)).
- intro. apply funextsec. intro t. induction t; reflexivity.
- intro a. apply pathsdirprod.
+ apply funextsec. apply homotrefl.
+ apply funextsec. apply homotrefl.
Theorem iscontrfunfromempty (X : UU) : iscontr (empty -> X).
Show proof.
Theorem iscontrfunfromempty2 (X : UU) {Y : UU} (is : neg Y) : iscontr (Y -> X).
Show proof.
intros. set (w := weqtoempty is). set (w' := weqbfun X (invweq w)).
apply (iscontrweqb w' (iscontrfunfromempty X)).
apply (iscontrweqb w' (iscontrfunfromempty X)).
Definition funfromcoprodtoprod {X Y Z : UU} (f : X ⨿ Y -> Z) :
(X -> Z) × (Y -> Z)
:= make_dirprod (λ x, f (ii1 x)) (λ y : Y, f (ii2 y)).
Definition prodtofunfromcoprod {X Y Z : UU} (fg : (X -> Z) × (Y -> Z)) :
X ⨿ Y -> Z := sumofmaps (pr1 fg) (pr2 fg).
Theorem weqfunfromcoprodtoprod (X Y Z : UU) :
(X ⨿ Y -> Z) ≃ ((X -> Z) × (Y -> Z)).
Show proof.
intros.
simple refine (
make_weq _ (isweq_iso (@funfromcoprodtoprod X Y Z)
(@prodtofunfromcoprod X Y Z) _ _)).
- intro a. apply funextfun; intro xy. induction xy as [ x | y ]; apply idpath.
- intro a. induction a as [fx fy]. apply idpath.
simple refine (
make_weq _ (isweq_iso (@funfromcoprodtoprod X Y Z)
(@prodtofunfromcoprod X Y Z) _ _)).
- intro a. apply funextfun; intro xy. induction xy as [ x | y ]; apply idpath.
- intro a. induction a as [fx fy]. apply idpath.
Definition tosecoverunit (P : unit -> UU) (p : P tt) : ∏ t : unit, P t.
Show proof.
intros. induction t. apply p.
Definition weqsecoverunit (P : unit -> UU) : (∏ t : unit, P t) ≃ (P tt).
Show proof.
set (f := λ a : ∏ t : unit, P t, a tt).
set (g := tosecoverunit P).
split with f.
assert (egf : ∏ a, g (f a) = a).
{
intro. apply funextsec.
intro t. induction t. apply idpath.
}
assert (efg : ∏ a, f (g a) = a) by (intros; apply idpath).
apply (isweq_iso _ _ egf efg).
set (g := tosecoverunit P).
split with f.
assert (egf : ∏ a, g (f a) = a).
{
intro. apply funextsec.
intro t. induction t. apply idpath.
}
assert (efg : ∏ a, f (g a) = a) by (intros; apply idpath).
apply (isweq_iso _ _ egf efg).
Definition weqsecovercontr {X : UU} (P : X -> UU) (is : iscontr X) :
(∏ x, P x) ≃ (P (pr1 is)).
Show proof.
Definition tosecovertotal2 {X : UU} (P : X -> UU) (Q : (∑ x, P x) -> UU)
(a : ∏ x, ∏ p : P x, Q (x ,, p)) :
∏ xp : (∑ x, P x), Q xp.
Show proof.
intros. induction xp as [ x p ]. apply (a x p).
General equivalence between curried and uncurried function types
Definition weqsecovertotal2 {X : UU} (P : X -> UU) (Q : (∑ x, P x) -> UU) :
(∏ xp : (∑ x, P x), Q xp) ≃ (∏ x, ∏ p : P x, Q (x,, p)).
Show proof.
(∏ xp : (∑ x, P x), Q xp) ≃ (∏ x, ∏ p : P x, Q (x,, p)).
Show proof.
intros.
set (f := λ a : ∏ xp : (∑ x, P x), Q xp, λ x, λ p : P x, a (x,, p)).
set (g := tosecovertotal2 P Q). split with f.
assert (egf : ∏ a, g (f a) = a).
{
intro. apply funextsec.
intro xp. induction xp as [ x p ]. apply idpath.
}
assert (efg : ∏ a, f (g a) = a).
{
intro. apply funextsec.
intro x. apply funextsec.
intro p. apply idpath.
}
apply (isweq_iso _ _ egf efg).
set (f := λ a : ∏ xp : (∑ x, P x), Q xp, λ x, λ p : P x, a (x,, p)).
set (g := tosecovertotal2 P Q). split with f.
assert (egf : ∏ a, g (f a) = a).
{
intro. apply funextsec.
intro xp. induction xp as [ x p ]. apply idpath.
}
assert (efg : ∏ a, f (g a) = a).
{
intro. apply funextsec.
intro x. apply funextsec.
intro p. apply idpath.
}
apply (isweq_iso _ _ egf efg).
Functions from unit and from contractible types
Definition weqfunfromunit (X : UU) : (unit -> X) ≃ X := weqsecoverunit _.
Definition weqfunfromcontr {X : UU} (Y : UU) (is : iscontr X) : (X -> Y) ≃ Y
:= weqsecovercontr _ is.
Functions from total2
Definition weqfunfromtotal2 {X : UU} (P : X -> UU) (Y : UU) :
((∑ x, P x) -> Y) ≃ (∏ x, P x -> Y) := weqsecovertotal2 P _.
Definition weqfunfromdirprod (X X' Y : UU) :
(X × X' -> Y) ≃ (∏ x, X' -> Y) := weqsecovertotal2 _ _.
Theorem saying that if each member of a family is of h-level n then the space of sections of the family is of h-level n.
General case
Theorem impred (n : nat) {T : UU} (P : T -> UU) :
(∏ t : T, isofhlevel n (P t)) -> (isofhlevel n (∏ t : T, P t)).
Show proof.
revert T P. induction n as [ | n IHn ].
- intros T P X. apply (funcontr P X).
- intros T P X. unfold isofhlevel in X. unfold isofhlevel. intros x x'.
assert (is : ∏ t : T, isofhlevel n (x t = x' t))
by (intro; apply (X t (x t) (x' t))).
assert (is2 : isofhlevel n (∏ t : T, x t = x' t))
by apply (IHn _ (λ t0 : T, x t0 = x' t0) is).
set (u := toforallpaths P x x').
assert (is3: isweq u) by apply isweqtoforallpaths.
set (v:= invmap (make_weq u is3)).
assert (is4: isweq v) by apply isweqinvmap.
apply (isofhlevelweqf n (make_weq v is4)).
assumption.
- intros T P X. apply (funcontr P X).
- intros T P X. unfold isofhlevel in X. unfold isofhlevel. intros x x'.
assert (is : ∏ t : T, isofhlevel n (x t = x' t))
by (intro; apply (X t (x t) (x' t))).
assert (is2 : isofhlevel n (∏ t : T, x t = x' t))
by apply (IHn _ (λ t0 : T, x t0 = x' t0) is).
set (u := toforallpaths P x x').
assert (is3: isweq u) by apply isweqtoforallpaths.
set (v:= invmap (make_weq u is3)).
assert (is4: isweq v) by apply isweqinvmap.
apply (isofhlevelweqf n (make_weq v is4)).
assumption.
Corollary impred_iscontr {T : UU} (P : T -> UU) :
(∏ t : T, iscontr (P t)) -> (iscontr (∏ t : T, P t)).
Show proof.
Corollary impred_isaprop {T : UU} (P : T -> UU) :
(∏ t : T, isaprop (P t)) -> (isaprop (∏ t : T, P t)).
Show proof.
Corollary impred_isaset {T : UU} (P : T -> UU) :
(∏ t : T, isaset (P t)) -> (isaset (∏ t : T, P t)).
Show proof.
Corollary impredtwice (n : nat) {T T' : UU} (P : T -> T' -> UU) :
(∏ (t : T) (t': T'), isofhlevel n (P t t'))
-> (isofhlevel n (∏ (t : T) (t': T'), P t t')).
Show proof.
intros X.
assert (is1 : ∏ t : T, isofhlevel n (∏ t': T', P t t'))
by (intro; apply (impred n _ (X t))).
apply (impred n _ is1).
assert (is1 : ∏ t : T, isofhlevel n (∏ t': T', P t t'))
by (intro; apply (impred n _ (X t))).
apply (impred n _ is1).
Corollary impredfun (n : nat) (X Y : UU) (is : isofhlevel n Y) :
isofhlevel n (X -> Y).
Show proof.
Theorem impredtech1 (n : nat) (X Y : UU) :
(X -> isofhlevel n Y) -> isofhlevel n (X -> Y).
Show proof.
revert X Y. induction n as [ | n IHn ]. intros X Y X0. simpl.
split with (λ x, pr1 (X0 x)).
- intro t.
assert (s1 : ∏ x, t x = pr1 (X0 x))
by (intro; apply proofirrelevancecontr; apply (X0 x)).
apply funextsec. assumption.
- intros X Y X0. simpl.
assert (X1 : X -> isofhlevel (S n) (X -> Y))
by (intro X1; apply impred; assumption).
intros x x'.
assert (s1 : isofhlevel n (∏ xx, x xx = x' xx))
by (apply impred; intro t; apply (X0 t)).
assert (w : (∏ xx, x xx = x' xx) ≃ (x = x'))
by apply (weqfunextsec _ x x').
apply (isofhlevelweqf n w s1).
split with (λ x, pr1 (X0 x)).
- intro t.
assert (s1 : ∏ x, t x = pr1 (X0 x))
by (intro; apply proofirrelevancecontr; apply (X0 x)).
apply funextsec. assumption.
- intros X Y X0. simpl.
assert (X1 : X -> isofhlevel (S n) (X -> Y))
by (intro X1; apply impred; assumption).
intros x x'.
assert (s1 : isofhlevel n (∏ xx, x xx = x' xx))
by (apply impred; intro t; apply (X0 t)).
assert (w : (∏ xx, x xx = x' xx) ≃ (x = x'))
by apply (weqfunextsec _ x x').
apply (isofhlevelweqf n w s1).
Theorem iscontrfuntounit (X : UU) : iscontr (X -> unit).
Show proof.
Theorem iscontrfuntocontr (X : UU) {Y : UU} (is : iscontr Y) : iscontr (X -> Y).
Show proof.
Functions to an empty type (generalization of isapropneg )
Theorem iscontriscontr {X : UU} (is : iscontr X) : iscontr (iscontr X).
Show proof.
assert (is0 : ∏ (x x' : X), x = x')
by (apply proofirrelevancecontr; assumption).
assert (is1 : ∏ cntr : X, iscontr (∏ x, x = cntr)).
{
intro.
assert (is2 : ∏ x, iscontr (x = cntr)).
{
assert (is2 : isaprop X)
by (apply isapropifcontr; assumption).
unfold isaprop in is2. unfold isofhlevel in is2.
intro x. apply (is2 x cntr).
}
apply funcontr. assumption.
}
set (f := @pr1 X (λ cntr : X, ∏ x, x = cntr)).
assert (X1 : isweq f)
by (apply isweqpr1; assumption).
change (∑ (cntr : X), ∏ x, x = cntr) with (iscontr X) in X1.
apply (iscontrweqb (make_weq f X1)). assumption.
by (apply proofirrelevancecontr; assumption).
assert (is1 : ∏ cntr : X, iscontr (∏ x, x = cntr)).
{
intro.
assert (is2 : ∏ x, iscontr (x = cntr)).
{
assert (is2 : isaprop X)
by (apply isapropifcontr; assumption).
unfold isaprop in is2. unfold isofhlevel in is2.
intro x. apply (is2 x cntr).
}
apply funcontr. assumption.
}
set (f := @pr1 X (λ cntr : X, ∏ x, x = cntr)).
assert (X1 : isweq f)
by (apply isweqpr1; assumption).
change (∑ (cntr : X), ∏ x, x = cntr) with (iscontr X) in X1.
apply (iscontrweqb (make_weq f X1)). assumption.
Theorem isapropiscontr (T : UU) : isaprop (iscontr T).
Show proof.
intros. unfold isaprop. unfold isofhlevel.
intros x x'. assert (is : iscontr(iscontr T)).
apply iscontriscontr. apply x.
assert (is2 : isaprop (iscontr T)) by apply (isapropifcontr is).
apply (is2 x x').
intros x x'. assert (is : iscontr(iscontr T)).
apply iscontriscontr. apply x.
assert (is2 : isaprop (iscontr T)) by apply (isapropifcontr is).
apply (is2 x x').
Theorem isapropisweq {X Y : UU} (f : X -> Y) : isaprop (isweq f).
Show proof.
intros. unfold isweq.
apply (impred (S O) (λ y : Y, iscontr (hfiber f y))
(λ y : Y, isapropiscontr (hfiber f y))).
apply (impred (S O) (λ y : Y, iscontr (hfiber f y))
(λ y : Y, isapropiscontr (hfiber f y))).
Theorem isapropisisolated (X : UU) (x : X) : isaprop (isisolated X x).
Show proof.
intros. apply isofhlevelsn. intro is. apply impred. intro x'.
apply (isapropdec _ (isaproppathsfromisolated X x is x')).
apply (isapropdec _ (isaproppathsfromisolated X x is x')).
Theorem isapropisdeceq (X : UU) : isaprop (isdeceq X).
Show proof.
apply (isofhlevelsn 0). intro is. unfold isdeceq. apply impred.
intro x. apply (isapropisisolated X x).
intro x. apply (isapropisisolated X x).
Theorem isapropisofhlevel (n : nat) (X : UU) : isaprop (isofhlevel n X).
Show proof.
revert X. induction n as [ | n IHn ].
- apply isapropiscontr.
- intro X.
apply impred. intros t.
apply impred. intros t0.
apply IHn.
- apply isapropiscontr.
- intro X.
apply impred. intros t.
apply impred. intros t0.
apply IHn.
Corollary isapropisaprop (X : UU) : isaprop (isaprop X).
Show proof.
Definition isapropisdecprop (X : UU) : isaprop (isdecprop X).
Show proof.
intros.
unfold isdecprop.
apply (isofhlevelweqf 1 (weqdirprodcomm _ _)).
apply isofhleveltotal2.
- apply isapropisaprop.
- intro i. apply isapropdec. assumption.
unfold isdecprop.
apply (isofhlevelweqf 1 (weqdirprodcomm _ _)).
apply isofhleveltotal2.
- apply isapropisaprop.
- intro i. apply isapropdec. assumption.
Corollary isapropisaset (X : UU) : isaprop (isaset X).
Show proof.
Theorem isapropisofhlevelf (n : nat) {X Y : UU} (f : X -> Y) :
isaprop (isofhlevelf n f).
Show proof.
Definition isapropisincl {X Y : UU} (f : X -> Y) : isaprop (isofhlevelf 1 f)
:= isapropisofhlevelf 1 f.
Lemma isaprop_isInjective {X Y : UU} (f : X -> Y) : isaprop (isInjective f).
Show proof.
Lemma incl_injectivity {X Y : UU} (f : X -> Y) : isincl f ≃ isInjective f.
Show proof.
intros.
apply weqimplimpl.
- apply isweqonpathsincl.
- apply isinclweqonpaths.
- apply isapropisincl.
- apply isaprop_isInjective.
apply weqimplimpl.
- apply isweqonpathsincl.
- apply isinclweqonpaths.
- apply isapropisincl.
- apply isaprop_isInjective.
Theorems saying that various pr1 maps are inclusions
Theorem isinclpr1weq (X Y : UU) : isincl (pr1weq : X ≃ Y -> X -> Y).
Show proof.
Corollary isinjpr1weq (X Y : UU) : isInjective (pr1weq : X ≃ Y -> X -> Y).
Show proof.
Theorem isinclpr1isolated (T : UU) : isincl (pr1isolated T).
Show proof.
associativity of weqcomp
Definition weqcomp_assoc {W X Y Z : UU} (f : W ≃ X) (g: X ≃ Y) (h : Y ≃ Z) :
(h ∘ (g ∘ f) = (h ∘ g) ∘ f)%weq.
Show proof.
Lemma eqweqmap_pathscomp0 {A B C : UU} (p : A = B) (q : B = C)
: weqcomp (eqweqmap p) (eqweqmap q)
= eqweqmap (pathscomp0 p q).
Show proof.
Lemma inv_idweq_is_idweq {A : UU} :
idweq A = invweq (idweq A).
Show proof.
Lemma eqweqmap_pathsinv0 {A B : UU} (p : A = B)
: eqweqmap (!p) = invweq (eqweqmap p).
Show proof.
Various weak equivalences between spaces of weak equivalences
Composition with a weak quivalence is a weak equivalence on weak equivalences
Theorem weqfweq (X : UU) {Y Z : UU} (w : Y ≃ Z) : (X ≃ Y) ≃ (X ≃ Z).
Show proof.
intros.
set (f := λ a : X ≃ Y, weqcomp a w).
set (g := λ b : X ≃ Z, weqcomp b (invweq w)).
split with f.
assert (egf : ∏ a, g (f a) = a).
{
intro a. apply (invmaponpathsincl _ (isinclpr1weq _ _)). apply funextfun.
intro x. apply (homotinvweqweq w (a x)).
}
assert (efg : ∏ b, f (g b) = b).
{
intro b. apply (invmaponpathsincl _ (isinclpr1weq _ _)). apply funextfun.
intro x. apply (homotweqinvweq w (b x)).
}
apply (isweq_iso _ _ egf efg).
set (f := λ a : X ≃ Y, weqcomp a w).
set (g := λ b : X ≃ Z, weqcomp b (invweq w)).
split with f.
assert (egf : ∏ a, g (f a) = a).
{
intro a. apply (invmaponpathsincl _ (isinclpr1weq _ _)). apply funextfun.
intro x. apply (homotinvweqweq w (a x)).
}
assert (efg : ∏ b, f (g b) = b).
{
intro b. apply (invmaponpathsincl _ (isinclpr1weq _ _)). apply funextfun.
intro x. apply (homotweqinvweq w (b x)).
}
apply (isweq_iso _ _ egf efg).
Theorem weqbweq {X Y : UU} (Z : UU) (w : X ≃ Y) : (Y ≃ Z) ≃ (X ≃ Z).
Show proof.
intros.
set (f := λ a : Y ≃ Z, weqcomp w a).
set (g := λ b : X ≃ Z, weqcomp (invweq w) b).
split with f.
assert (egf : ∏ a, g (f a) = a).
{
intro a. apply (invmaponpathsincl _ (isinclpr1weq _ _)). apply funextfun.
intro y. apply (maponpaths a (homotweqinvweq w y)).
}
assert (efg : ∏ b, f (g b) = b).
{
intro b. apply (invmaponpathsincl _ (isinclpr1weq _ _)). apply funextfun.
intro x. apply (maponpaths b (homotinvweqweq w x)).
}
apply (isweq_iso _ _ egf efg).
set (f := λ a : Y ≃ Z, weqcomp w a).
set (g := λ b : X ≃ Z, weqcomp (invweq w) b).
split with f.
assert (egf : ∏ a, g (f a) = a).
{
intro a. apply (invmaponpathsincl _ (isinclpr1weq _ _)). apply funextfun.
intro y. apply (maponpaths a (homotweqinvweq w y)).
}
assert (efg : ∏ b, f (g b) = b).
{
intro b. apply (invmaponpathsincl _ (isinclpr1weq _ _)). apply funextfun.
intro x. apply (maponpaths b (homotinvweqweq w x)).
}
apply (isweq_iso _ _ egf efg).
Theorem weqweq {X Y : UU} (w: X ≃ Y) : (X ≃ X) ≃ (Y ≃ Y).
Show proof.
intros. intermediate_weq (X ≃ Y).
- apply weqfweq. assumption.
- apply invweq. apply weqbweq. assumption.
- apply weqfweq. assumption.
- apply invweq. apply weqbweq. assumption.
Invertion on weak equivalences as a weak equivalence
Theorem weqinvweq (X Y : UU) : (X ≃ Y) ≃ (Y ≃ X).
Show proof.
intros.
apply (weq_iso invweq invweq).
- intro. apply (invmaponpathsincl _ (isinclpr1weq _ _)). apply funextfun. apply homotrefl.
- intro. apply (invmaponpathsincl _ (isinclpr1weq _ _)). apply funextfun. apply homotrefl.
apply (weq_iso invweq invweq).
- intro. apply (invmaponpathsincl _ (isinclpr1weq _ _)). apply funextfun. apply homotrefl.
- intro. apply (invmaponpathsincl _ (isinclpr1weq _ _)). apply funextfun. apply homotrefl.
Theorem isofhlevelsnweqtohlevelsn (n : nat) (X Y : UU)
(is : isofhlevel (S n) Y) : isofhlevel (S n) (X ≃ Y).
Show proof.
Theorem isofhlevelsnweqfromhlevelsn (n : nat) (X Y : UU)
(is : isofhlevel (S n) Y) : isofhlevel (S n) (Y ≃ X).
Show proof.
Theorem isapropweqtocontr (X : UU) {Y : UU} (is : iscontr Y) : isaprop (X ≃ Y).
Show proof.
Theorem isapropweqfromcontr (X : UU) {Y : UU} (is : iscontr Y) : isaprop (Y ≃ X).
Show proof.
Theorem isapropweqtoprop (X Y : UU) (is : isaprop Y) : isaprop (X ≃ Y).
Show proof.
Theorem isapropweqfromprop (X Y : UU) (is : isaprop Y) : isaprop (Y ≃ X).
Show proof.
Theorem isasetweqtoset (X Y : UU) (is : isaset Y) : isaset (X ≃ Y).
Show proof.
Theorem isasetweqfromset (X Y : UU) (is : isaset Y) : isaset (Y ≃ X).
Show proof.
Theorem isapropweqtoempty (X : UU) : isaprop (X ≃ empty).
Show proof.
Theorem isapropweqtoempty2 (X : UU) {Y : UU} (is : neg Y) : isaprop (X ≃ Y).
Show proof.
Theorem isapropweqfromempty (X : UU) : isaprop (empty ≃ X).
Show proof.
Theorem isapropweqfromempty2 (X : UU) {Y : UU} (is : neg Y) : isaprop (Y ≃ X).
Show proof.
Weak equivalences to and from unit
Theorem isapropweqtounit (X : UU) : isaprop (X ≃ unit).
Show proof.
Theorem isapropweqfromunit (X : UU) : isaprop (unit ≃ X).
Show proof.
Definition cutonweq {T : UU} t (is : isisolated T t) (w : T ≃ T) :
isolated T × (compl T t ≃ compl T t).
Show proof.
intros. split.
- exists (w t). apply isisolatedweqf. assumption.
- intermediate_weq (compl T (w t)).
+ apply weqoncompl.
+ apply weqtranspos0.
* apply isisolatedweqf. assumption.
* assumption.
- exists (w t). apply isisolatedweqf. assumption.
- intermediate_weq (compl T (w t)).
+ apply weqoncompl.
+ apply weqtranspos0.
* apply isisolatedweqf. assumption.
* assumption.
Definition invcutonweq {T : UU} (t : T)
(is : isisolated T t)
(t'w : isolated T × (compl T t ≃ compl T t)) : T ≃ T
:= weqcomp (weqrecomplf t t is is (pr2 t'w))
(weqtranspos t (pr1 (pr1 t'w)) is (pr2 (pr1 t'w))).
Lemma pathsinvcuntonweqoft {T : UU} (t : T)
(is : isisolated T t)
(t'w : isolated T × (compl T t ≃ compl T t)) :
invcutonweq t is t'w t = pr1 (pr1 t'w).
Show proof.
intros. unfold invcutonweq. simpl. unfold recompl. unfold coprodf.
unfold invmap. simpl. unfold invrecompl.
induction (is t) as [ ett | nett ].
- apply pathsfuntransposoft1.
- induction (nett (idpath _)).
unfold invmap. simpl. unfold invrecompl.
induction (is t) as [ ett | nett ].
- apply pathsfuntransposoft1.
- induction (nett (idpath _)).
Definition weqcutonweq (T : UU) (t : T) (is : isisolated T t) :
(T ≃ T) ≃ isolated T × (compl T t ≃ compl T t).
Show proof.
intros.
set (f := cutonweq t is). set (g := invcutonweq t is).
apply (weq_iso f g).
- intro w. Set Printing Coercions. idtac.
apply (invmaponpathsincl _ (isinclpr1weq _ _)).
apply funextfun; intro t'. simpl.
unfold invmap; simpl. unfold coprodf, invrecompl.
induction (is t') as [ ett' | nett' ].
+ simpl. rewrite (pathsinv0 ett'). apply pathsfuntransposoft1.
+ unfold funtranspos0; simpl.
induction (is (w t)) as [ etwt | netwt ].
* induction (is (w t')) as [ etwt' | netwt' ].
-- induction (negf (invmaponpathsincl w (isofhlevelfweq 1 w) t t') nett'
(pathscomp0 (pathsinv0 etwt) etwt')).
-- simpl. assert (newtt'' := netwt'). rewrite etwt in netwt'.
apply (pathsfuntransposofnet1t2 t (w t) is _ (w t') newtt'' netwt').
* simpl. induction (is (w t')) as [ etwt' | netwt' ].
-- simpl. rewrite (pathsinv0 etwt').
apply (pathsfuntransposoft2 t (w t) is _).
-- simpl.
assert (ne : neg (w t = w t'))
by apply (negf (invmaponpathsweq w _ _) nett').
apply (pathsfuntransposofnet1t2 t (w t) is _ (w t') netwt' ne).
- intro xw. induction xw as [ x w ]. induction x as [ t' is' ].
simpl in w. apply pathsdirprod.
+ apply (invmaponpathsincl _ (isinclpr1isolated _)).
simpl. unfold recompl, coprodf, invmap; simpl. unfold invrecompl.
induction (is t) as [ ett | nett ].
* apply pathsfuntransposoft1.
* induction (nett (idpath _)).
+ simpl.
apply (invmaponpathsincl _ (isinclpr1weq _ _) _ _). apply funextfun.
intro x. induction x as [ x netx ].
unfold g, invcutonweq; simpl.
set (int := funtranspos
(t,, is) (t',, is')
(recompl T t (coprodf w (λ x0 :unit, x0)
(invmap (weqrecompl T t is) t)))).
assert (eee : int = t').
{
unfold int. unfold recompl, coprodf, invmap; simpl. unfold invrecompl.
induction (is t) as [ ett | nett ].
- apply pathsfuntransposoft1.
- induction (nett (idpath _)).
}
assert (isint : isisolated _ int).
{
rewrite eee. apply is'.
}
apply (ishomotinclrecomplf _ _ isint (funtranspos0 _ _ _) _ _).
simpl.
change (recomplf int t isint (funtranspos0 int t is))
with (funtranspos (int,, isint) (t,, is)).
assert (ee : (int,, isint) = (t',, is')).
{
apply (invmaponpathsincl _ (isinclpr1isolated _) _ _).
simpl. apply eee.
}
rewrite ee.
set (e := homottranspost2t1t1t2
t t' is is'
(recompl T t (coprodf w (λ x0 : unit, x0)
(invmap (weqrecompl T t is) x)))).
simpl in e.
rewrite e. unfold recompl, coprodf, invmap; simpl. unfold invrecompl.
induction (is x) as [ etx | netx' ].
* induction (netx etx).
* apply (maponpaths (@pr1 _ _)). apply (maponpaths w).
apply (invmaponpathsincl _ (isinclpr1compl _ _) _ _).
simpl. apply idpath.
Unset Printing Coercions.
set (f := cutonweq t is). set (g := invcutonweq t is).
apply (weq_iso f g).
- intro w. Set Printing Coercions. idtac.
apply (invmaponpathsincl _ (isinclpr1weq _ _)).
apply funextfun; intro t'. simpl.
unfold invmap; simpl. unfold coprodf, invrecompl.
induction (is t') as [ ett' | nett' ].
+ simpl. rewrite (pathsinv0 ett'). apply pathsfuntransposoft1.
+ unfold funtranspos0; simpl.
induction (is (w t)) as [ etwt | netwt ].
* induction (is (w t')) as [ etwt' | netwt' ].
-- induction (negf (invmaponpathsincl w (isofhlevelfweq 1 w) t t') nett'
(pathscomp0 (pathsinv0 etwt) etwt')).
-- simpl. assert (newtt'' := netwt'). rewrite etwt in netwt'.
apply (pathsfuntransposofnet1t2 t (w t) is _ (w t') newtt'' netwt').
* simpl. induction (is (w t')) as [ etwt' | netwt' ].
-- simpl. rewrite (pathsinv0 etwt').
apply (pathsfuntransposoft2 t (w t) is _).
-- simpl.
assert (ne : neg (w t = w t'))
by apply (negf (invmaponpathsweq w _ _) nett').
apply (pathsfuntransposofnet1t2 t (w t) is _ (w t') netwt' ne).
- intro xw. induction xw as [ x w ]. induction x as [ t' is' ].
simpl in w. apply pathsdirprod.
+ apply (invmaponpathsincl _ (isinclpr1isolated _)).
simpl. unfold recompl, coprodf, invmap; simpl. unfold invrecompl.
induction (is t) as [ ett | nett ].
* apply pathsfuntransposoft1.
* induction (nett (idpath _)).
+ simpl.
apply (invmaponpathsincl _ (isinclpr1weq _ _) _ _). apply funextfun.
intro x. induction x as [ x netx ].
unfold g, invcutonweq; simpl.
set (int := funtranspos
(t,, is) (t',, is')
(recompl T t (coprodf w (λ x0 :unit, x0)
(invmap (weqrecompl T t is) t)))).
assert (eee : int = t').
{
unfold int. unfold recompl, coprodf, invmap; simpl. unfold invrecompl.
induction (is t) as [ ett | nett ].
- apply pathsfuntransposoft1.
- induction (nett (idpath _)).
}
assert (isint : isisolated _ int).
{
rewrite eee. apply is'.
}
apply (ishomotinclrecomplf _ _ isint (funtranspos0 _ _ _) _ _).
simpl.
change (recomplf int t isint (funtranspos0 int t is))
with (funtranspos (int,, isint) (t,, is)).
assert (ee : (int,, isint) = (t',, is')).
{
apply (invmaponpathsincl _ (isinclpr1isolated _) _ _).
simpl. apply eee.
}
rewrite ee.
set (e := homottranspost2t1t1t2
t t' is is'
(recompl T t (coprodf w (λ x0 : unit, x0)
(invmap (weqrecompl T t is) x)))).
simpl in e.
rewrite e. unfold recompl, coprodf, invmap; simpl. unfold invrecompl.
induction (is x) as [ etx | netx' ].
* induction (netx etx).
* apply (maponpaths (@pr1 _ _)). apply (maponpaths w).
apply (invmaponpathsincl _ (isinclpr1compl _ _) _ _).
simpl. apply idpath.
Unset Printing Coercions.
some lemmas about weak equivalences
Definition weqcompidl {X Y} (f:X ≃ Y) : weqcomp (idweq X) f = f.
Show proof.
intros. apply (invmaponpathsincl _ (isinclpr1weq _ _)).
apply funextsec; intro x; simpl. apply idpath.
apply funextsec; intro x; simpl. apply idpath.
Definition weqcompidr {X Y} (f:X ≃ Y) : weqcomp f (idweq Y) = f.
Show proof.
intros. apply (invmaponpathsincl _ (isinclpr1weq _ _)).
apply funextsec; intro x; simpl. apply idpath.
apply funextsec; intro x; simpl. apply idpath.
Definition weqcompinvl {X Y} (f:X ≃ Y) : weqcomp (invweq f) f = idweq Y.
Show proof.
intros. apply (invmaponpathsincl _ (isinclpr1weq _ _)).
apply funextsec; intro y; simpl. apply homotweqinvweq.
apply funextsec; intro y; simpl. apply homotweqinvweq.
Definition weqcompinvr {X Y} (f:X ≃ Y) : weqcomp f (invweq f) = idweq X.
Show proof.
intros. apply (invmaponpathsincl _ (isinclpr1weq _ _)).
apply funextsec; intro x; simpl. apply homotinvweqweq.
apply funextsec; intro x; simpl. apply homotinvweqweq.
Definition weqcompassoc {X Y Z W} (f:X ≃ Y) (g:Y ≃ Z) (h:Z ≃ W) :
weqcomp (weqcomp f g) h = weqcomp f (weqcomp g h).
Show proof.
intros. apply (invmaponpathsincl _ (isinclpr1weq _ _)).
apply funextsec; intro x; simpl. apply idpath.
apply funextsec; intro x; simpl. apply idpath.
Definition weqcompweql {X Y Z} (f:X ≃ Y) :
isweq (λ g:Y ≃ Z, weqcomp f g).
Show proof.
intros. simple refine (isweq_iso _ _ _ _).
{ intro h. exact (weqcomp (invweq f) h). }
{ intro g. simpl. rewrite <- weqcompassoc. rewrite weqcompinvl. apply weqcompidl. }
{ intro h. simpl. rewrite <- weqcompassoc. rewrite weqcompinvr. apply weqcompidl. }
{ intro h. exact (weqcomp (invweq f) h). }
{ intro g. simpl. rewrite <- weqcompassoc. rewrite weqcompinvl. apply weqcompidl. }
{ intro h. simpl. rewrite <- weqcompassoc. rewrite weqcompinvr. apply weqcompidl. }
Definition weqcompweqr {X Y Z} (g:Y ≃ Z) :
isweq (λ f:X ≃ Y, weqcomp f g).
Show proof.
intros. simple refine (isweq_iso _ _ _ _).
{ intro h. exact (weqcomp h (invweq g)). }
{ intro f. simpl. rewrite weqcompassoc. rewrite weqcompinvr. apply weqcompidr. }
{ intro h. simpl. rewrite weqcompassoc. rewrite weqcompinvl. apply weqcompidr. }
{ intro h. exact (weqcomp h (invweq g)). }
{ intro f. simpl. rewrite weqcompassoc. rewrite weqcompinvr. apply weqcompidr. }
{ intro h. simpl. rewrite weqcompassoc. rewrite weqcompinvl. apply weqcompidr. }
Definition weqcompinjr {X Y Z} {f f':X ≃ Y} (g:Y ≃ Z) :
weqcomp f g = weqcomp f' g -> f = f'.
Show proof.
Definition weqcompinjl {X Y Z} (f:X ≃ Y) {g g':Y ≃ Z} :
weqcomp f g = weqcomp f g' -> g = g'.
Show proof.
Definition invweqcomp {X Y Z} (f:X ≃ Y) (g:Y ≃ Z) :
invweq (weqcomp f g) = weqcomp (invweq g) (invweq f).
Show proof.
intros. apply (weqcompinjr (weqcomp f g)). rewrite weqcompinvl.
rewrite weqcompassoc. rewrite <- (weqcompassoc (invweq f)).
rewrite weqcompinvl. rewrite weqcompidl. rewrite weqcompinvl. apply idpath.
rewrite weqcompassoc. rewrite <- (weqcompassoc (invweq f)).
rewrite weqcompinvl. rewrite weqcompidl. rewrite weqcompinvl. apply idpath.
Definition invmapweqcomp {X Y Z} (f:X ≃ Y) (g:Y ≃ Z) :
invmap (weqcomp f g) = weqcomp (invweq g) (invweq f).
Show proof.
reflexivity.