Library UniMath.CategoryTheory.elems_slice_equiv
**********************************************************
Matthew Weaver, 2017
**********************************************************
Contents : Equivalence of the categories PreShv ∫P and
PreShv C / P for any P in PreShv C
Require Import UniMath.Foundations.Sets.
Require Import UniMath.MoreFoundations.Tactics.
Require Import UniMath.CategoryTheory.Core.Categories.
Require Import UniMath.CategoryTheory.Core.Isos.
Require Import UniMath.CategoryTheory.Core.Functors.
Require Import UniMath.CategoryTheory.Core.NaturalTransformations.
Require Import UniMath.CategoryTheory.FunctorCategory.
Require Import
UniMath.CategoryTheory.Equivalences.Core
UniMath.CategoryTheory.categories.HSET.Core
UniMath.CategoryTheory.categories.HSET.MonoEpiIso
UniMath.CategoryTheory.slicecat
UniMath.CategoryTheory.opp_precat
UniMath.CategoryTheory.Presheaf
UniMath.CategoryTheory.ElementsOp.
Section elems_slice_equiv.
Local Open Scope cat.
Local Notation "C / X" := (slice_cat C X).
Local Definition ap_PreShv {X : category} := fun (P : PreShv X) (x : X) => pr1hSet ((pr1 P) x).
Local Notation "##" := ap_PreShv.
Variable (C : category) (P : PreShv C).
Local Open Scope cat.
Local Notation "C / X" := (slice_cat C X).
Local Definition ap_PreShv {X : category} := fun (P : PreShv X) (x : X) => pr1hSet ((pr1 P) x).
Local Notation "##" := ap_PreShv.
Variable (C : category) (P : PreShv C).
Local Definition make_ob := @make_ob C P.
Local Definition make_mor := @make_mor C P.
Definition PreShv_to_slice_ob_funct_fun (F : PreShv ∫P) : C^op → HSET :=
λ X, total2_hSet (fun p : ##P X => (pr1 F) (make_ob X p)).
Definition PreShv_to_slice_ob_funct_mor (F : PreShv ∫P) {X Y : C^op} (f : X --> Y) :
PreShv_to_slice_ob_funct_fun F X --> PreShv_to_slice_ob_funct_fun F Y :=
λ p, # (pr1 P) f (pr1 p) ,, # (pr1 F) (mor_to_el_mor (C:=C) f (pr1 p)) (pr2 p).
Definition PreShv_to_slice_ob_funct_data (F : PreShv ∫P) : functor_data C^op HSET :=
PreShv_to_slice_ob_funct_fun F ,, @PreShv_to_slice_ob_funct_mor F.
Definition PreShv_to_slice_ob_is_funct (F : PreShv ∫P) : is_functor (PreShv_to_slice_ob_funct_data F).
Show proof.
Definition PreShv_to_slice_ob_is_funct' (F : PreShv ∫P) : is_functor (PreShv_to_slice_ob_funct_data F).
Show proof.
Definition PreShv_to_slice_ob_funct (F : PreShv ∫P) : PreShv C :=
PreShv_to_slice_ob_funct_data F ,, PreShv_to_slice_ob_is_funct F.
Definition PreShv_to_slice_ob_nat_fun (F : PreShv ∫P) (x : C) : (∑ (Px :##P x), ##F (x,, Px)) → ##P x := pr1.
Definition PreShv_to_slice_ob : PreShv ∫P → PreShv C / P.
Show proof.
Definition PreShv_to_slice_ob_nat {X Y : PreShv ∫P} (f : X --> Y) (c : C)
: (∑ Px : ## P c, ## X (c,, Px)) → (∑ Px : ## P c, ## Y (c,, Px)) :=
λ p, pr1 p ,, (pr1 f) (c ,, (pr1 p)) (pr2 p).
Definition PreShv_to_slice_ob_isnat {X Y : PreShv ∫P} (f : X --> Y) :
is_nat_trans (PreShv_to_slice_ob_funct_data X) (PreShv_to_slice_ob_funct_data Y) (PreShv_to_slice_ob_nat f).
simpl.
intros c c' g.
apply funextsec; intro p.
apply pair_path_in2.
exact (eqtohomot ((pr2 f) (c ,, pr1 p) (c',, # (pr1 P) g (pr1 p)) (g,, idpath (# (pr1 P) g (pr1 p)))) (pr2 p)).
Qed.
Definition PreShv_to_slice_mor {X Y : PreShv ∫P} (f : X --> Y) :
PreShv_to_slice_ob X --> PreShv_to_slice_ob Y.
exists (PreShv_to_slice_ob_nat f ,, PreShv_to_slice_ob_isnat f).
now apply (nat_trans_eq has_homsets_HSET).
Defined.
Definition PreShv_to_slice_data : functor_data (PreShv ∫P) (PreShv C / P) :=
PreShv_to_slice_ob ,, @PreShv_to_slice_mor.
Definition PreShv_to_slice_is_funct : is_functor PreShv_to_slice_data.
Show proof.
Definition PreShv_to_slice : functor (PreShv ∫P) (PreShv C / P) :=
PreShv_to_slice_data ,, PreShv_to_slice_is_funct.
Local Definition make_mor := @make_mor C P.
Definition PreShv_to_slice_ob_funct_fun (F : PreShv ∫P) : C^op → HSET :=
λ X, total2_hSet (fun p : ##P X => (pr1 F) (make_ob X p)).
Definition PreShv_to_slice_ob_funct_mor (F : PreShv ∫P) {X Y : C^op} (f : X --> Y) :
PreShv_to_slice_ob_funct_fun F X --> PreShv_to_slice_ob_funct_fun F Y :=
λ p, # (pr1 P) f (pr1 p) ,, # (pr1 F) (mor_to_el_mor (C:=C) f (pr1 p)) (pr2 p).
Definition PreShv_to_slice_ob_funct_data (F : PreShv ∫P) : functor_data C^op HSET :=
PreShv_to_slice_ob_funct_fun F ,, @PreShv_to_slice_ob_funct_mor F.
Definition PreShv_to_slice_ob_is_funct (F : PreShv ∫P) : is_functor (PreShv_to_slice_ob_funct_data F).
Show proof.
split.
+ intros I; apply funextfun; intros [ρ u].
use total2_paths_f.
* exact (eqtohomot (functor_id P I) ρ).
* etrans; [use transportf_make_ob|].
etrans; [apply transportf_PreShv|]; cbn.
now rewrite (mor_to_el_mor_id ρ), transportfbinv, (functor_id F).
+ intros I J K f g; apply funextfun; intros [ρ u].
use total2_paths_f.
* exact (eqtohomot (functor_comp P f g) ρ).
* etrans; [use transportf_make_ob|].
etrans; [apply transportf_PreShv|].
rewrite (mor_to_el_mor_comp _ f g), transportfbinv.
generalize u; simpl in *.
apply eqtohomot, (functor_comp F (mor_to_el_mor f ρ) (mor_to_el_mor g (# (pr1 P) f ρ))).
+ intros I; apply funextfun; intros [ρ u].
use total2_paths_f.
* exact (eqtohomot (functor_id P I) ρ).
* etrans; [use transportf_make_ob|].
etrans; [apply transportf_PreShv|]; cbn.
now rewrite (mor_to_el_mor_id ρ), transportfbinv, (functor_id F).
+ intros I J K f g; apply funextfun; intros [ρ u].
use total2_paths_f.
* exact (eqtohomot (functor_comp P f g) ρ).
* etrans; [use transportf_make_ob|].
etrans; [apply transportf_PreShv|].
rewrite (mor_to_el_mor_comp _ f g), transportfbinv.
generalize u; simpl in *.
apply eqtohomot, (functor_comp F (mor_to_el_mor f ρ) (mor_to_el_mor g (# (pr1 P) f ρ))).
Definition PreShv_to_slice_ob_is_funct' (F : PreShv ∫P) : is_functor (PreShv_to_slice_ob_funct_data F).
Show proof.
split;
[intros X | intros X Y Z f g];
apply funextsec; intros [p q].
+ set (T := ∑ p' : ## P X, p' = # (pr1 P) (identity X) p : UU).
set (T' := ∑ p' : ## P X, (pr1 F) (X ,, p) --> (pr1 F) (X ,, p') : UU).
set (phi := λ (x : T), make_mor (X ,, pr1 x) (X ,, p) (identity X) (pr2 x)).
set (G := λ (x : T), pr1 x ,, # (pr1 F) (phi x) : T').
set (e := fun (x : ∫P) => eqtohomot (!((functor_id P) (pr1 x))) (pr2 x)).
set (h := λ (x : T'), pr1 x ,, (pr2 x) q : pr1hSet (PreShv_to_slice_ob_funct_fun F X)).
use (maponpaths (funcomp G h)
(coconustot_isProofIrrelevant ((# (pr1 P) (identity X) p) ,, idpath _) (p ,, e (X ,, p))) @ _).
use (@pair_path_in2 _ (λ x, pr1hSet ((pr1 F) (X ,, x))) p).
use (eqtohomot _ q @ eqtohomot (functor_id F (X ,, p)) q).
use (maponpaths (# (pr1 F))).
use total2_paths_f.
* reflexivity.
* rewrite idpath_transportf;
now apply setproperty.
+ set (T := ∑ p' : ## P Z, p' = # (pr1 P) (g ∘ f) p : UU).
set (T' := ∑ p' : ## P Z, (pr1 F) (X ,, p) --> (pr1 F) (Z ,, p') : UU).
set (phi := λ (x : T), make_mor (Z ,, pr1 x) (X ,, p) (g ∘ f) (pr2 x)).
set (G := λ (x : T), (pr1 x ,, # (pr1 F) (phi x)) : T').
set (e := fun (z y x : ∫P) (f : z --> y) (g : y --> x) =>
((pr2 f) @ maponpaths (# (pr1 P) (pr1 f)) (pr2 g)
@ (eqtohomot (!(functor_comp P) (pr1 g) (pr1 f)) (pr2 x)))).
set (h := λ (x : T'), pr1 x ,, (pr2 x) q : pr1hSet (PreShv_to_slice_ob_funct_fun F Z)).
use (maponpaths (funcomp G h)
(coconustot_isProofIrrelevant (# (pr1 P) (g ∘ f) p ,, idpath _)
(# (pr1 P) g (# (pr1 P) f p) ,,
e (make_ob Z (# (pr1 P) g (# (pr1 P) f p)))
(make_ob Y (# (pr1 P) f p)) (make_ob X p)
(g ,, idpath _) (f ,, idpath _))) @ _).
use (@pair_path_in2 _ (λ x, pr1hSet ((pr1 F) (Z ,, x))) (# (pr1 P) g (# (pr1 P) f p))).
use (eqtohomot _ q @ eqtohomot (@functor_comp _ _ F (make_ob X p)
(make_ob Y (# (pr1 P) f p))
(make_ob Z (# (pr1 P) g (# (pr1 P) f p)))
(f ,, idpath _) (g,, idpath _)) q).
use (maponpaths (# (pr1 F))).
use total2_paths_f.
* reflexivity.
* rewrite idpath_transportf;
now apply setproperty.
[intros X | intros X Y Z f g];
apply funextsec; intros [p q].
+ set (T := ∑ p' : ## P X, p' = # (pr1 P) (identity X) p : UU).
set (T' := ∑ p' : ## P X, (pr1 F) (X ,, p) --> (pr1 F) (X ,, p') : UU).
set (phi := λ (x : T), make_mor (X ,, pr1 x) (X ,, p) (identity X) (pr2 x)).
set (G := λ (x : T), pr1 x ,, # (pr1 F) (phi x) : T').
set (e := fun (x : ∫P) => eqtohomot (!((functor_id P) (pr1 x))) (pr2 x)).
set (h := λ (x : T'), pr1 x ,, (pr2 x) q : pr1hSet (PreShv_to_slice_ob_funct_fun F X)).
use (maponpaths (funcomp G h)
(coconustot_isProofIrrelevant ((# (pr1 P) (identity X) p) ,, idpath _) (p ,, e (X ,, p))) @ _).
use (@pair_path_in2 _ (λ x, pr1hSet ((pr1 F) (X ,, x))) p).
use (eqtohomot _ q @ eqtohomot (functor_id F (X ,, p)) q).
use (maponpaths (# (pr1 F))).
use total2_paths_f.
* reflexivity.
* rewrite idpath_transportf;
now apply setproperty.
+ set (T := ∑ p' : ## P Z, p' = # (pr1 P) (g ∘ f) p : UU).
set (T' := ∑ p' : ## P Z, (pr1 F) (X ,, p) --> (pr1 F) (Z ,, p') : UU).
set (phi := λ (x : T), make_mor (Z ,, pr1 x) (X ,, p) (g ∘ f) (pr2 x)).
set (G := λ (x : T), (pr1 x ,, # (pr1 F) (phi x)) : T').
set (e := fun (z y x : ∫P) (f : z --> y) (g : y --> x) =>
((pr2 f) @ maponpaths (# (pr1 P) (pr1 f)) (pr2 g)
@ (eqtohomot (!(functor_comp P) (pr1 g) (pr1 f)) (pr2 x)))).
set (h := λ (x : T'), pr1 x ,, (pr2 x) q : pr1hSet (PreShv_to_slice_ob_funct_fun F Z)).
use (maponpaths (funcomp G h)
(coconustot_isProofIrrelevant (# (pr1 P) (g ∘ f) p ,, idpath _)
(# (pr1 P) g (# (pr1 P) f p) ,,
e (make_ob Z (# (pr1 P) g (# (pr1 P) f p)))
(make_ob Y (# (pr1 P) f p)) (make_ob X p)
(g ,, idpath _) (f ,, idpath _))) @ _).
use (@pair_path_in2 _ (λ x, pr1hSet ((pr1 F) (Z ,, x))) (# (pr1 P) g (# (pr1 P) f p))).
use (eqtohomot _ q @ eqtohomot (@functor_comp _ _ F (make_ob X p)
(make_ob Y (# (pr1 P) f p))
(make_ob Z (# (pr1 P) g (# (pr1 P) f p)))
(f ,, idpath _) (g,, idpath _)) q).
use (maponpaths (# (pr1 F))).
use total2_paths_f.
* reflexivity.
* rewrite idpath_transportf;
now apply setproperty.
Definition PreShv_to_slice_ob_funct (F : PreShv ∫P) : PreShv C :=
PreShv_to_slice_ob_funct_data F ,, PreShv_to_slice_ob_is_funct F.
Definition PreShv_to_slice_ob_nat_fun (F : PreShv ∫P) (x : C) : (∑ (Px :##P x), ##F (x,, Px)) → ##P x := pr1.
Definition PreShv_to_slice_ob : PreShv ∫P → PreShv C / P.
Show proof.
Definition PreShv_to_slice_ob_nat {X Y : PreShv ∫P} (f : X --> Y) (c : C)
: (∑ Px : ## P c, ## X (c,, Px)) → (∑ Px : ## P c, ## Y (c,, Px)) :=
λ p, pr1 p ,, (pr1 f) (c ,, (pr1 p)) (pr2 p).
Definition PreShv_to_slice_ob_isnat {X Y : PreShv ∫P} (f : X --> Y) :
is_nat_trans (PreShv_to_slice_ob_funct_data X) (PreShv_to_slice_ob_funct_data Y) (PreShv_to_slice_ob_nat f).
simpl.
intros c c' g.
apply funextsec; intro p.
apply pair_path_in2.
exact (eqtohomot ((pr2 f) (c ,, pr1 p) (c',, # (pr1 P) g (pr1 p)) (g,, idpath (# (pr1 P) g (pr1 p)))) (pr2 p)).
Qed.
Definition PreShv_to_slice_mor {X Y : PreShv ∫P} (f : X --> Y) :
PreShv_to_slice_ob X --> PreShv_to_slice_ob Y.
exists (PreShv_to_slice_ob_nat f ,, PreShv_to_slice_ob_isnat f).
now apply (nat_trans_eq has_homsets_HSET).
Defined.
Definition PreShv_to_slice_data : functor_data (PreShv ∫P) (PreShv C / P) :=
PreShv_to_slice_ob ,, @PreShv_to_slice_mor.
Definition PreShv_to_slice_is_funct : is_functor PreShv_to_slice_data.
Show proof.
split; [intros X | intros X Y Z f g];
apply eq_mor_slicecat;
apply (nat_trans_eq has_homsets_HSET);
unfold PreShv_to_slice_ob_nat , PreShv_to_slice_ob_funct_fun;
intro c;
apply funextsec; intro p;
reflexivity.
apply eq_mor_slicecat;
apply (nat_trans_eq has_homsets_HSET);
unfold PreShv_to_slice_ob_nat , PreShv_to_slice_ob_funct_fun;
intro c;
apply funextsec; intro p;
reflexivity.
Definition PreShv_to_slice : functor (PreShv ∫P) (PreShv C / P) :=
PreShv_to_slice_data ,, PreShv_to_slice_is_funct.
Definition slice_to_PreShv_ob_ob (Q : PreShv C / P) : (∫P)^op → HSET :=
λ p,
hfiber ((pr1 (pr2 Q)) (pr1 p)) (pr2 p) ,,
isaset_hfiber ((pr1 (pr2 Q)) (pr1 p)) (pr2 p) (pr2 (((pr1 (pr1 Q)) (pr1 p)))) (pr2 ((pr1 P) (pr1 p))).
Definition slice_to_PreShv_ob_mor (Q : PreShv C / P) {F G : (∫P)^op} (f : F --> G) :
slice_to_PreShv_ob_ob Q F --> slice_to_PreShv_ob_ob Q G.
intros s.
destruct Q as [[[Q Qmor] Qisfunct] [Qnat Qisnat]].
destruct F as [x Px]. destruct G as [y Py].
destruct f as [f feq].
apply (hfibersgftog (Qmor _ _ f) (Qnat y)).
exists (pr1 s).
rewrite feq.
use (eqtohomot (Qisnat _ _ f) (pr1 s) @ _).
exact (maponpaths (# (pr1 P) f) (pr2 s)).
Defined.
Definition slice_to_PreShv_ob_funct_data (Q : PreShv C / P) : functor_data ((∫P)^op) HSET :=
slice_to_PreShv_ob_ob Q ,, @slice_to_PreShv_ob_mor Q.
Definition slice_to_PreShv_ob_is_funct (Q : PreShv C / P) : is_functor (slice_to_PreShv_ob_funct_data Q).
Show proof.
Definition slice_to_PreShv_ob : PreShv C / P → PreShv ∫P :=
λ Q, slice_to_PreShv_ob_funct_data Q ,, slice_to_PreShv_ob_is_funct Q.
Definition slice_to_PreShv_ob_nat {X Y : PreShv C / P} (F : X --> Y) (e : ∫P^op) :
(slice_to_PreShv_ob_ob X) e --> (slice_to_PreShv_ob_ob Y) e.
Show proof.
Definition slice_to_PreShv_ob_is_nat {X Y : PreShv C / P} (F : X --> Y) :
is_nat_trans (slice_to_PreShv_ob X : functor _ _) (slice_to_PreShv_ob Y : functor _ _) (slice_to_PreShv_ob_nat F).
Show proof.
Definition slice_to_PreShv_mor {X Y : PreShv C / P} (F : X --> Y) :
slice_to_PreShv_ob X --> slice_to_PreShv_ob Y :=
slice_to_PreShv_ob_nat F ,, slice_to_PreShv_ob_is_nat F.
Definition slice_to_PreShv_data : functor_data (PreShv C / P) (PreShv ∫P) :=
slice_to_PreShv_ob ,, @slice_to_PreShv_mor.
Definition slice_to_PreShv_is_funct : is_functor slice_to_PreShv_data.
Show proof.
Definition slice_to_PreShv : functor (PreShv C / P) (PreShv ∫P) :=
slice_to_PreShv_data ,, slice_to_PreShv_is_funct.
λ p,
hfiber ((pr1 (pr2 Q)) (pr1 p)) (pr2 p) ,,
isaset_hfiber ((pr1 (pr2 Q)) (pr1 p)) (pr2 p) (pr2 (((pr1 (pr1 Q)) (pr1 p)))) (pr2 ((pr1 P) (pr1 p))).
Definition slice_to_PreShv_ob_mor (Q : PreShv C / P) {F G : (∫P)^op} (f : F --> G) :
slice_to_PreShv_ob_ob Q F --> slice_to_PreShv_ob_ob Q G.
intros s.
destruct Q as [[[Q Qmor] Qisfunct] [Qnat Qisnat]].
destruct F as [x Px]. destruct G as [y Py].
destruct f as [f feq].
apply (hfibersgftog (Qmor _ _ f) (Qnat y)).
exists (pr1 s).
rewrite feq.
use (eqtohomot (Qisnat _ _ f) (pr1 s) @ _).
exact (maponpaths (# (pr1 P) f) (pr2 s)).
Defined.
Definition slice_to_PreShv_ob_funct_data (Q : PreShv C / P) : functor_data ((∫P)^op) HSET :=
slice_to_PreShv_ob_ob Q ,, @slice_to_PreShv_ob_mor Q.
Definition slice_to_PreShv_ob_is_funct (Q : PreShv C / P) : is_functor (slice_to_PreShv_ob_funct_data Q).
Show proof.
split;
[intros [x Px] | intros [x Px] [y Py] [z Pz] [f feq] [g geq]];
destruct Q as [[[Q Qmor] Qisfunct] [Qnat Qisnat]];
apply funextsec; intro p;
apply (invmaponpathsincl pr1);
try (apply isofhlevelfpr1;
intro; apply setproperty).
+ exact (eqtohomot ((pr1 Qisfunct) x) (pr1 p)).
+ exact (eqtohomot ((pr2 Qisfunct) x y z f g) (pr1 p)).
[intros [x Px] | intros [x Px] [y Py] [z Pz] [f feq] [g geq]];
destruct Q as [[[Q Qmor] Qisfunct] [Qnat Qisnat]];
apply funextsec; intro p;
apply (invmaponpathsincl pr1);
try (apply isofhlevelfpr1;
intro; apply setproperty).
+ exact (eqtohomot ((pr1 Qisfunct) x) (pr1 p)).
+ exact (eqtohomot ((pr2 Qisfunct) x y z f g) (pr1 p)).
Definition slice_to_PreShv_ob : PreShv C / P → PreShv ∫P :=
λ Q, slice_to_PreShv_ob_funct_data Q ,, slice_to_PreShv_ob_is_funct Q.
Definition slice_to_PreShv_ob_nat {X Y : PreShv C / P} (F : X --> Y) (e : ∫P^op) :
(slice_to_PreShv_ob_ob X) e --> (slice_to_PreShv_ob_ob Y) e.
Show proof.
induction e as [e Pe].
exact (λ p, hfibersgftog ((pr1 (pr1 F)) e)
((pr1 (pr2 Y)) e) Pe
(transportf (λ x, hfiber (x e) Pe) (base_paths _ _ (pr2 F)) p)).
exact (λ p, hfibersgftog ((pr1 (pr1 F)) e)
((pr1 (pr2 Y)) e) Pe
(transportf (λ x, hfiber (x e) Pe) (base_paths _ _ (pr2 F)) p)).
Definition slice_to_PreShv_ob_is_nat {X Y : PreShv C / P} (F : X --> Y) :
is_nat_trans (slice_to_PreShv_ob X : functor _ _) (slice_to_PreShv_ob Y : functor _ _) (slice_to_PreShv_ob_nat F).
Show proof.
intros [e Pe] [e' Pe'] [f feq].
destruct X as [[[X Xmor] Xisfunct] [Xnat Xisnat]].
destruct Y as [[[Y Ymor] Yisfunct] [Ynat Yisnat]].
destruct F as [[F Fisnat] Feq].
simpl in *.
apply funextsec; intros [p peq].
apply (invmaponpathsincl pr1).
+ apply isofhlevelfpr1.
intro.
apply setproperty.
+ simpl.
destruct peq.
unfold hfiber.
repeat rewrite transportf_total2.
simpl.
repeat rewrite transportf_const.
exact (eqtohomot (Fisnat e e' f) p).
destruct X as [[[X Xmor] Xisfunct] [Xnat Xisnat]].
destruct Y as [[[Y Ymor] Yisfunct] [Ynat Yisnat]].
destruct F as [[F Fisnat] Feq].
simpl in *.
apply funextsec; intros [p peq].
apply (invmaponpathsincl pr1).
+ apply isofhlevelfpr1.
intro.
apply setproperty.
+ simpl.
destruct peq.
unfold hfiber.
repeat rewrite transportf_total2.
simpl.
repeat rewrite transportf_const.
exact (eqtohomot (Fisnat e e' f) p).
Definition slice_to_PreShv_mor {X Y : PreShv C / P} (F : X --> Y) :
slice_to_PreShv_ob X --> slice_to_PreShv_ob Y :=
slice_to_PreShv_ob_nat F ,, slice_to_PreShv_ob_is_nat F.
Definition slice_to_PreShv_data : functor_data (PreShv C / P) (PreShv ∫P) :=
slice_to_PreShv_ob ,, @slice_to_PreShv_mor.
Definition slice_to_PreShv_is_funct : is_functor slice_to_PreShv_data.
Show proof.
split; [ intros X | intros X Y Z F G];
apply (nat_trans_eq has_homsets_HSET);
intros [c Pc];
apply funextsec; intros [p peq];
apply (invmaponpathsincl pr1);
try (apply isofhlevelfpr1;
intro;
apply setproperty);
simpl;
unfold hfiber;
unfold hfibersgftog; unfold make_hfiber;
repeat (rewrite transportf_total2;
simpl; unfold hfiber);
now repeat rewrite transportf_const.
apply (nat_trans_eq has_homsets_HSET);
intros [c Pc];
apply funextsec; intros [p peq];
apply (invmaponpathsincl pr1);
try (apply isofhlevelfpr1;
intro;
apply setproperty);
simpl;
unfold hfiber;
unfold hfibersgftog; unfold make_hfiber;
repeat (rewrite transportf_total2;
simpl; unfold hfiber);
now repeat rewrite transportf_const.
Definition slice_to_PreShv : functor (PreShv C / P) (PreShv ∫P) :=
slice_to_PreShv_data ,, slice_to_PreShv_is_funct.
Construction of the natural isomorphism from (slice_to_PreShv ∙ PreShv_to_slice) to the identity functor
Definition slice_counit_fun (X : PreShv C / P) :
(slice_to_PreShv ∙ PreShv_to_slice) X --> (functor_identity _) X.
Show proof.
Definition is_nat_trans_slice_counit : is_nat_trans _ _ slice_counit_fun.
Show proof.
Definition slice_counit : slice_to_PreShv ∙ PreShv_to_slice ⟹ functor_identity (PreShv C / P) :=
slice_counit_fun ,, is_nat_trans_slice_counit.
Definition slice_all_z_iso : forall F : PreShv C / P, is_z_isomorphism (slice_counit F).
Show proof.
Definition slice_unit : functor_identity (PreShv C / P) ⟹ slice_to_PreShv ∙ PreShv_to_slice :=
pr1 (nat_trafo_z_iso_if_pointwise_z_iso (has_homsets_slice_precat ((PreShv C)) P) (slice_counit) slice_all_z_iso).
(slice_to_PreShv ∙ PreShv_to_slice) X --> (functor_identity _) X.
Show proof.
destruct X as [[[X Xmor] Xisfunct] [Xnat Xisnat]].
simpl in *.
repeat (use tpair; simpl).
+ intros x [p q].
exact (pr1 q).
+ intros A B f.
apply funextsec; intros [p peq].
reflexivity.
+ apply (nat_trans_eq has_homsets_HSET).
intros A.
apply funextsec; intros [p [q e]].
exact (!e).
simpl in *.
repeat (use tpair; simpl).
+ intros x [p q].
exact (pr1 q).
+ intros A B f.
apply funextsec; intros [p peq].
reflexivity.
+ apply (nat_trans_eq has_homsets_HSET).
intros A.
apply funextsec; intros [p [q e]].
exact (!e).
Definition is_nat_trans_slice_counit : is_nat_trans _ _ slice_counit_fun.
Show proof.
intros X Y f.
apply eq_mor_slicecat , (nat_trans_eq has_homsets_HSET).
intros A.
apply funextsec; intros [p [q e]].
simpl. unfold compose. simpl.
destruct X as [[[X Xmor] Xisfunct] [Xnat Xisnat]].
destruct Y as [[[Y Ymor] Yisfunct] [Ynat Yisnat]].
destruct f as [[f fisnat] feq]. simpl in *.
apply maponpaths. unfold hfiber.
rewrite transportf_total2. simpl.
rewrite transportf_const.
reflexivity.
apply eq_mor_slicecat , (nat_trans_eq has_homsets_HSET).
intros A.
apply funextsec; intros [p [q e]].
simpl. unfold compose. simpl.
destruct X as [[[X Xmor] Xisfunct] [Xnat Xisnat]].
destruct Y as [[[Y Ymor] Yisfunct] [Ynat Yisnat]].
destruct f as [[f fisnat] feq]. simpl in *.
apply maponpaths. unfold hfiber.
rewrite transportf_total2. simpl.
rewrite transportf_const.
reflexivity.
Definition slice_counit : slice_to_PreShv ∙ PreShv_to_slice ⟹ functor_identity (PreShv C / P) :=
slice_counit_fun ,, is_nat_trans_slice_counit.
Definition slice_all_z_iso : forall F : PreShv C / P, is_z_isomorphism (slice_counit F).
Show proof.
intros [[[F Fmor] Fisfunct] [Fnat Fisnat]].
apply z_iso_to_slice_precat_z_iso.
apply nat_trafo_z_iso_if_pointwise_z_iso.
intros X; simpl.
change (λ X0, pr1 (pr2 X0)) with (fromcoconusf (Fnat X)).
exact (hset_equiv_is_z_iso (make_hSet (coconusf (Fnat X))
(isaset_total2_hSet _ (λ y, (hfiber_hSet (Fnat X) y)))) _
(weqfromcoconusf (Fnat X))).
apply z_iso_to_slice_precat_z_iso.
apply nat_trafo_z_iso_if_pointwise_z_iso.
intros X; simpl.
change (λ X0, pr1 (pr2 X0)) with (fromcoconusf (Fnat X)).
exact (hset_equiv_is_z_iso (make_hSet (coconusf (Fnat X))
(isaset_total2_hSet _ (λ y, (hfiber_hSet (Fnat X) y)))) _
(weqfromcoconusf (Fnat X))).
Definition slice_unit : functor_identity (PreShv C / P) ⟹ slice_to_PreShv ∙ PreShv_to_slice :=
pr1 (nat_trafo_z_iso_if_pointwise_z_iso (has_homsets_slice_precat ((PreShv C)) P) (slice_counit) slice_all_z_iso).
Construction of the natural isomorphism from the identity functor to (PreShv_to_slice ∙ slice_to_PreShv)
Definition PreShv_unit_fun (F : PreShv ∫P) :
(functor_identity _) F --> (PreShv_to_slice ∙ slice_to_PreShv) F.
Show proof.
Definition is_nat_trans_PreShv_unit : is_nat_trans _ _ PreShv_unit_fun.
Show proof.
Definition PreShv_unit : functor_identity (PreShv ∫P) ⟹ PreShv_to_slice ∙ slice_to_PreShv :=
PreShv_unit_fun ,, is_nat_trans_PreShv_unit.
Definition PreShv_all_iso : forall F : PreShv ∫P, is_z_isomorphism (PreShv_unit F).
Show proof.
Definition PreShv_counit : PreShv_to_slice ∙ slice_to_PreShv ⟹ functor_identity (PreShv ∫P) :=
pr1 (nat_trafo_z_iso_if_pointwise_z_iso (pr2 (PreShv ∫P)) PreShv_unit PreShv_all_iso).
(functor_identity _) F --> (PreShv_to_slice ∙ slice_to_PreShv) F.
Show proof.
use tpair.
+ intros [X p] x.
exact ((p ,, x) ,, idpath p).
+ intros [X p] [X' p'] [f feq].
simpl in *.
apply funextsec; intros x.
apply (invmaponpathsincl pr1).
apply isofhlevelfpr1;
intro;
apply setproperty.
induction (!feq).
apply (total2_paths2_f (idpath _)).
rewrite idpath_transportf.
assert (set_eq : idpath _ = feq).
{ apply (pr2 (P X')). }
now induction set_eq.
+ intros [X p] x.
exact ((p ,, x) ,, idpath p).
+ intros [X p] [X' p'] [f feq].
simpl in *.
apply funextsec; intros x.
apply (invmaponpathsincl pr1).
apply isofhlevelfpr1;
intro;
apply setproperty.
induction (!feq).
apply (total2_paths2_f (idpath _)).
rewrite idpath_transportf.
assert (set_eq : idpath _ = feq).
{ apply (pr2 (P X')). }
now induction set_eq.
Definition is_nat_trans_PreShv_unit : is_nat_trans _ _ PreShv_unit_fun.
Show proof.
intros [[F Fmor] Fisfunct] [[G Gmor] Gisfunct] [f fisnat].
apply (nat_trans_eq has_homsets_HSET).
intros [X p].
apply funextsec; intros q.
apply (invmaponpathsincl pr1).
apply isofhlevelfpr1;
intro;
apply setproperty.
simpl. unfold hfiber.
rewrite transportf_total2; simpl.
now rewrite transportf_const.
apply (nat_trans_eq has_homsets_HSET).
intros [X p].
apply funextsec; intros q.
apply (invmaponpathsincl pr1).
apply isofhlevelfpr1;
intro;
apply setproperty.
simpl. unfold hfiber.
rewrite transportf_total2; simpl.
now rewrite transportf_const.
Definition PreShv_unit : functor_identity (PreShv ∫P) ⟹ PreShv_to_slice ∙ slice_to_PreShv :=
PreShv_unit_fun ,, is_nat_trans_PreShv_unit.
Definition PreShv_all_iso : forall F : PreShv ∫P, is_z_isomorphism (PreShv_unit F).
Show proof.
intros [[F Fmor] Fisfunct].
apply nat_trafo_z_iso_if_pointwise_z_iso.
intros [X p]; simpl.
assert (H : isweq (λ x : pr1hSet (F (X,, p)) , (p,, x) ,, idpath p : pr1hSet (slice_to_PreShv_ob_ob (PreShv_to_slice_ob ((F,, Fmor),, Fisfunct)) (X,, p)))).
{ unfold isweq. intros [[p' x'] e'].
simpl in *. induction e'.
use ((x',, idpath _),, _).
intros [x'' t].
apply (invmaponpathsincl pr1).
apply isofhlevelfpr1;
intro;
exact (pr2 (@eqset
((slice_to_PreShv_ob_ob (PreShv_to_slice_ob ((F,, Fmor),, Fisfunct)) (X,, p'))) _ _)).
assert (eq_id : base_paths (p',, x'') (p',, x') (maponpaths pr1 t) = idpath p').
{ set (c := iscontraprop1 (setproperty _ _ _) (idpath p')).
exact ((pr2 c) _ @ !((pr2 c) _)).
}
set (eq := fiber_paths (maponpaths pr1 t)).
use (_ @ eq).
rewrite (transportf_paths _ eq_id).
now rewrite idpath_transportf.
}
exact (hset_equiv_is_z_iso (F (X ,, p)) _ (_ ,, H)).
apply nat_trafo_z_iso_if_pointwise_z_iso.
intros [X p]; simpl.
assert (H : isweq (λ x : pr1hSet (F (X,, p)) , (p,, x) ,, idpath p : pr1hSet (slice_to_PreShv_ob_ob (PreShv_to_slice_ob ((F,, Fmor),, Fisfunct)) (X,, p)))).
{ unfold isweq. intros [[p' x'] e'].
simpl in *. induction e'.
use ((x',, idpath _),, _).
intros [x'' t].
apply (invmaponpathsincl pr1).
apply isofhlevelfpr1;
intro;
exact (pr2 (@eqset
((slice_to_PreShv_ob_ob (PreShv_to_slice_ob ((F,, Fmor),, Fisfunct)) (X,, p'))) _ _)).
assert (eq_id : base_paths (p',, x'') (p',, x') (maponpaths pr1 t) = idpath p').
{ set (c := iscontraprop1 (setproperty _ _ _) (idpath p')).
exact ((pr2 c) _ @ !((pr2 c) _)).
}
set (eq := fiber_paths (maponpaths pr1 t)).
use (_ @ eq).
rewrite (transportf_paths _ eq_id).
now rewrite idpath_transportf.
}
exact (hset_equiv_is_z_iso (F (X ,, p)) _ (_ ,, H)).
Definition PreShv_counit : PreShv_to_slice ∙ slice_to_PreShv ⟹ functor_identity (PreShv ∫P) :=
pr1 (nat_trafo_z_iso_if_pointwise_z_iso (pr2 (PreShv ∫P)) PreShv_unit PreShv_all_iso).
Definition PreShv_of_elems_slice_of_PreShv_equiv : equivalence_of_cats (PreShv ∫P) (PreShv C / P) :=
(PreShv_to_slice ,, slice_to_PreShv ,, PreShv_unit ,, slice_counit) ,, (PreShv_all_iso ,, slice_all_z_iso).
Definition PreShv_of_elems_slice_of_PreShv_adj_equiv : adj_equivalence_of_cats PreShv_to_slice :=
@adjointification (PreShv ∫P) (PreShv C / P) PreShv_of_elems_slice_of_PreShv_equiv.
End elems_slice_equiv.
(PreShv_to_slice ,, slice_to_PreShv ,, PreShv_unit ,, slice_counit) ,, (PreShv_all_iso ,, slice_all_z_iso).
Definition PreShv_of_elems_slice_of_PreShv_adj_equiv : adj_equivalence_of_cats PreShv_to_slice :=
@adjointification (PreShv ∫P) (PreShv C / P) PreShv_of_elems_slice_of_PreShv_equiv.
End elems_slice_equiv.