Spectral/higher_groups.hlean

456 lines
18 KiB
Text
Raw Normal View History

/-
Copyright (c) 2015 Ulrik Buchholtz, Egbert Rijke and Floris van Doorn. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Ulrik Buchholtz, Egbert Rijke, Floris van Doorn
Formalization of the higher groups paper
-/
import .homotopy.EM
open eq is_conn pointed is_trunc trunc equiv is_equiv trunc_index susp nat algebra
prod.ops sigma sigma.ops category EM
namespace higher_group
2018-01-17 23:43:50 +00:00
set_option pp.binder_types true
2018-01-19 15:07:28 +00:00
universe variable u
2018-01-30 21:11:13 +00:00
/- Results not necessarily about higher groups which we repeat here, because they are mentioned in
the higher group paper -/
namespace hide
open pushout
definition connect_intro_pequiv {k : } {B : Type*} (A : Type*) (H : is_conn k B) :
ppmap B (connect k A) ≃* ppmap B A :=
is_conn.connect_intro_pequiv A H
2018-01-30 21:11:13 +00:00
definition is_conn_fun_prod_of_wedge (n m : ) (A B : Type*)
[cA : is_conn n A] [cB : is_conn m B] : is_conn_fun (m + n) (@prod_of_wedge A B) :=
is_conn_fun_prod_of_wedge n m A B
definition is_trunc_ppi_of_is_conn (k n : ) (X : Type*) (H : is_conn (k.-1) X)
(Y : X → Type*) (H3 : Πx, is_trunc (k + n) (Y x)) :
is_trunc n (Π*(x : X), Y x) :=
is_conn.is_trunc_ppi_of_is_conn _ (k.-2) H _ _ (le_of_eq (sub_one_add_plus_two_sub_one k n)⁻¹) _ H3
2018-01-30 21:11:13 +00:00
end hide
2018-01-31 18:01:17 +00:00
/- The k-groupal n-types.
We require that the carrier has a point (preserved by the equivalence) -/
2018-01-18 19:50:26 +00:00
2018-01-31 18:01:17 +00:00
structure GType (n k : ) : Type := /- (n,k)GType, denoted here as [n;k]GType -/
2018-01-18 19:50:26 +00:00
(car : ptrunctype.{u} n)
2018-01-19 15:07:28 +00:00
(B : pconntype.{u} (k.-1)) /- this is Bᵏ -/
2018-01-18 19:50:26 +00:00
(e : car ≃* Ω[k] B)
2018-01-31 18:01:17 +00:00
structure InfGType (k : ) : Type := /- (∞,k)GType, denoted here as [∞;k]GType -/
2018-01-18 19:50:26 +00:00
(car : pType.{u})
2018-01-19 15:07:28 +00:00
(B : pconntype.{u} (k.-1)) /- this is Bᵏ -/
2018-01-18 19:50:26 +00:00
(e : car ≃* Ω[k] B)
2018-01-31 18:01:17 +00:00
structure ωGType (n : ) := /- (n,ω)GType, denoted here as [n;ω]GType -/
2018-01-18 19:50:26 +00:00
(B : Π(k : ), (n+k)-Type*[k.-1])
(e : Π(k : ), B k ≃* Ω (B (k+1)))
2018-01-31 18:01:17 +00:00
attribute InfGType.car GType.car [coercion]
2018-01-18 19:50:26 +00:00
2018-02-01 02:39:01 +00:00
variables {n k k' l : }
2018-01-31 18:01:17 +00:00
notation `[`:95 n:0 `; ` k `]GType`:0 := GType n k
notation `[∞; `:95 k:0 `]GType`:0 := InfGType k
notation `[`:95 n:0 `;ω]GType`:0 := ωGType n
2018-01-18 19:50:26 +00:00
2018-01-31 18:01:17 +00:00
open GType
open InfGType (renaming B→iB e→ie)
open ωGType (renaming B→oB e→oe)
2018-01-18 19:50:26 +00:00
/- some basic properties -/
2018-01-31 18:01:17 +00:00
lemma is_trunc_B' (G : [n;k]GType) : is_trunc (k+n) (B G) :=
2018-01-18 19:50:26 +00:00
begin
apply is_trunc_of_is_trunc_loopn,
2018-09-07 14:30:39 +00:00
exact is_trunc_equiv_closed _ (e G) _,
2018-01-18 19:50:26 +00:00
exact _
end
2018-01-31 18:01:17 +00:00
lemma is_trunc_B (G : [n;k]GType) : is_trunc (n+k) (B G) :=
2018-01-18 19:50:26 +00:00
transport (λm, is_trunc m (B G)) (add.comm k n) (is_trunc_B' G)
local attribute [instance] is_trunc_B
2018-01-31 18:01:17 +00:00
definition GType.sigma_char (n k : ) :
GType.{u} n k ≃ Σ(B : pconntype.{u} (k.-1)), Σ(X : ptrunctype.{u} n), X ≃* Ω[k] B :=
2018-01-19 15:07:28 +00:00
begin
fapply equiv.MK,
{ intro G, exact ⟨B G, G, e G⟩ },
2018-01-31 18:01:17 +00:00
{ intro v, exact GType.mk v.2.1 v.1 v.2.2 },
2018-01-19 15:07:28 +00:00
{ intro v, induction v with v₁ v₂, induction v₂, reflexivity },
{ intro G, induction G, reflexivity },
end
2018-01-31 18:01:17 +00:00
definition GType_equiv (n k : ) : [n;k]GType ≃ (n+k)-Type*[k.-1] :=
GType.sigma_char n k ⬝e
sigma_equiv_of_is_embedding_left_contr
ptruncconntype.to_pconntype
(is_embedding_ptruncconntype_to_pconntype (n+k) (k.-1))
begin
intro X,
apply is_trunc_equiv_closed_rev -2,
{ apply sigma_equiv_sigma_right, intro B',
refine _ ⬝e (ptrunctype_eq_equiv B' (ptrunctype.mk (Ω[k] X) !is_trunc_loopn_nat pt))⁻¹ᵉ,
assert lem : Π(A : n-Type*) (B : Type*) (H : is_trunc n B),
(A ≃* B) ≃ (A ≃* (ptrunctype.mk B H pt)),
{ intro A B'' H, induction B'', reflexivity },
2018-09-07 14:30:39 +00:00
apply lem },
exact _
end
begin
2018-01-31 18:01:17 +00:00
intro B' H, apply fiber.mk (ptruncconntype.mk B' (is_trunc_B (GType.mk H.1 B' H.2)) pt _),
induction B' with G' B' e', reflexivity
end
2018-01-18 19:50:26 +00:00
2018-01-31 18:01:17 +00:00
definition GType_equiv_pequiv {n k : } (G : [n;k]GType) : GType_equiv n k G ≃* B G :=
by reflexivity
2018-01-18 19:50:26 +00:00
2018-01-31 18:01:17 +00:00
definition GType_eq_equiv {n k : } (G H : [n;k]GType) : (G = H :> [n;k]GType) ≃ (B G ≃* B H) :=
2018-09-07 14:30:39 +00:00
eq_equiv_fn_eq (GType_equiv n k) _ _ ⬝e !ptruncconntype_eq_equiv
2018-01-19 15:07:28 +00:00
2018-01-31 18:01:17 +00:00
definition GType_eq {n k : } {G H : [n;k]GType} (e : B G ≃* B H) : G = H :=
(GType_eq_equiv G H)⁻¹ᵉ e
2018-01-18 19:50:26 +00:00
2018-01-31 18:01:17 +00:00
/- similar properties for [∞;k]GType -/
2018-01-31 18:01:17 +00:00
definition InfGType.sigma_char (k : ) :
InfGType.{u} k ≃ Σ(B : pconntype.{u} (k.-1)), Σ(X : pType.{u}), X ≃* Ω[k] B :=
begin
fapply equiv.MK,
{ intro G, exact ⟨iB G, G, ie G⟩ },
2018-01-31 18:01:17 +00:00
{ intro v, exact InfGType.mk v.2.1 v.1 v.2.2 },
{ intro v, induction v with v₁ v₂, induction v₂, reflexivity },
{ intro G, induction G, reflexivity },
end
2018-01-31 18:01:17 +00:00
definition InfGType_equiv (k : ) : [∞;k]GType ≃ Type*[k.-1] :=
InfGType.sigma_char k ⬝e
@sigma_equiv_of_is_contr_right _ _
2018-09-07 14:30:39 +00:00
(λX, is_trunc_equiv_closed_rev -2 (sigma_equiv_sigma_right (λB', !pType_eq_equiv⁻¹ᵉ)) _)
2018-01-31 18:01:17 +00:00
definition InfGType_equiv_pequiv {k : } (G : [∞;k]GType) : InfGType_equiv k G ≃* iB G :=
by reflexivity
2018-01-31 18:01:17 +00:00
definition InfGType_eq_equiv {k : } (G H : [∞;k]GType) : (G = H :> [∞;k]GType) ≃ (iB G ≃* iB H) :=
2018-09-07 14:30:39 +00:00
eq_equiv_fn_eq (InfGType_equiv k) _ _ ⬝e !pconntype_eq_equiv
2018-01-31 18:01:17 +00:00
definition InfGType_eq {k : } {G H : [∞;k]GType} (e : iB G ≃* iB H) : G = H :=
(InfGType_eq_equiv G H)⁻¹ᵉ e
2018-01-18 19:50:26 +00:00
2018-02-01 02:39:01 +00:00
/- alternative constructor for ωGType -/
definition ωGType.mk_le {n : } (k₀ : )
(C : Π⦃k : ℕ⦄, k₀ ≤ k → ((n+k)-Type*[k.-1] : Type.{u+1}))
(e : Π⦃k : ℕ⦄ (H : k₀ ≤ k), C H ≃* Ω (C (le.step H))) : ([n;ω]GType : Type.{u+1}) :=
begin
fconstructor,
{ apply rec_down_le _ k₀ C, intro n' D,
refine (ptruncconntype.mk (Ω D) _ pt _),
apply is_trunc_loop, apply is_trunc_ptruncconntype, apply is_conn_loop,
apply is_conn_ptruncconntype },
{ intro n', apply rec_down_le_univ, exact e, intro n D, reflexivity }
end
definition ωGType.mk_le_beta {n : } {k₀ : }
(C : Π⦃k : ℕ⦄, k₀ ≤ k → ((n+k)-Type*[k.-1] : Type.{u+1}))
(e : Π⦃k : ℕ⦄ (H : k₀ ≤ k), C H ≃* Ω (C (le.step H)))
(k : ) (H : k₀ ≤ k) : oB (ωGType.mk_le k₀ C e) k ≃* C H :=
ptruncconntype_eq_equiv _ _ !rec_down_le_beta_ge
definition GType_hom (G H : [n;k]GType) : Type :=
B G →* B H
definition ωGType_hom (G H : [n;ω]GType) : Type* :=
pointed.MK
(Σ(f : Πn, oB G n →* oB H n), Πn, psquare (f n) (Ω→ (f (n+1))) (oe G n) (oe H n))
⟨λn, pconst (oB G n) (oB H n), λn, !phconst_square ⬝vp* !ap1_pconst⟩
2018-01-18 19:50:26 +00:00
/- Constructions on higher groups -/
2018-01-31 18:01:17 +00:00
definition Decat (G : [n+1;k]GType) : [n;k]GType :=
GType.mk (ptrunctype.mk (ptrunc n G) _ pt) (pconntype.mk (ptrunc (n + k) (B G)) _ pt)
2018-01-18 19:50:26 +00:00
abstract begin
refine ptrunc_pequiv_ptrunc n (e G) ⬝e* _,
2018-01-19 15:07:28 +00:00
symmetry, exact !loopn_ptrunc_pequiv_nat
2018-01-18 19:50:26 +00:00
end end
2018-01-31 18:01:17 +00:00
definition Disc (G : [n;k]GType) : [n+1;k]GType :=
GType.mk (ptrunctype.mk G (show is_trunc (n.+1) G, from _) pt) (B G) (e G)
2018-01-18 19:50:26 +00:00
2018-01-31 18:01:17 +00:00
definition Decat_adjoint_Disc (G : [n+1;k]GType) (H : [n;k]GType) :
2018-01-18 19:50:26 +00:00
ppmap (B (Decat G)) (B H) ≃* ppmap (B G) (B (Disc H)) :=
pmap_ptrunc_pequiv (n + k) (B G) (B H)
2018-01-31 18:01:17 +00:00
definition Decat_adjoint_Disc_natural {G G' : [n+1;k]GType} {H H' : [n;k]GType}
(g : B G' →* B G) (h : B H →* B H') :
2018-01-18 19:50:26 +00:00
psquare (Decat_adjoint_Disc G H)
(Decat_adjoint_Disc G' H')
(ppcompose_left h ∘* ppcompose_right (ptrunc_functor _ g))
(ppcompose_left h ∘* ppcompose_right g) :=
pmap_ptrunc_pequiv_natural (n + k) g h
2018-01-18 19:50:26 +00:00
2018-01-31 18:01:17 +00:00
definition Decat_Disc (G : [n;k]GType) : Decat (Disc G) = G :=
GType_eq !ptrunc_pequiv
2018-01-18 19:50:26 +00:00
2018-01-31 18:01:17 +00:00
definition InfDecat (n : ) (G : [∞;k]GType) : [n;k]GType :=
GType.mk (ptrunctype.mk (ptrunc n G) _ pt) (pconntype.mk (ptrunc (n + k) (iB G)) _ pt)
2018-01-18 19:50:26 +00:00
abstract begin
refine ptrunc_pequiv_ptrunc n (ie G) ⬝e* _,
symmetry, exact !loopn_ptrunc_pequiv_nat
end end
2018-01-31 18:01:17 +00:00
definition InfDisc (n : ) (G : [n;k]GType) : [∞;k]GType :=
InfGType.mk G (B G) (e G)
2018-01-18 19:50:26 +00:00
2018-01-31 18:01:17 +00:00
definition InfDecat_adjoint_InfDisc (G : [∞;k]GType) (H : [n;k]GType) :
2018-01-18 19:50:26 +00:00
ppmap (B (InfDecat n G)) (B H) ≃* ppmap (iB G) (iB (InfDisc n H)) :=
pmap_ptrunc_pequiv (n + k) (iB G) (B H)
2018-02-01 02:39:01 +00:00
definition InfDecat_adjoint_InfDisc_natural {G G' : [∞;k]GType} {H H' : [n;k]GType}
(g : iB G' →* iB G) (h : B H →* B H') :
psquare (InfDecat_adjoint_InfDisc G H)
(InfDecat_adjoint_InfDisc G' H')
(ppcompose_left h ∘* ppcompose_right (ptrunc_functor _ g))
(ppcompose_left h ∘* ppcompose_right g) :=
pmap_ptrunc_pequiv_natural (n + k) g h
2018-01-18 19:50:26 +00:00
2018-01-31 18:01:17 +00:00
definition InfDecat_InfDisc (G : [n;k]GType) : InfDecat n (InfDisc n G) = G :=
GType_eq !ptrunc_pequiv
2018-01-18 19:50:26 +00:00
2018-01-31 18:01:17 +00:00
definition Deloop (G : [n;k+1]GType) : [n+1;k]GType :=
2018-01-18 19:50:26 +00:00
have is_conn k (B G), from is_conn_pconntype (B G),
have is_trunc (n + (k + 1)) (B G), from is_trunc_B G,
have is_trunc ((n + 1) + k) (B G), from transport (λ(n : ), is_trunc n _) (succ_add n k)⁻¹ this,
2018-01-31 18:01:17 +00:00
GType.mk (ptrunctype.mk (Ω[k] (B G)) !is_trunc_loopn_nat pt)
2018-01-18 19:50:26 +00:00
(pconntype.mk (B G) !is_conn_of_is_conn_succ pt)
(pequiv_of_equiv erfl idp)
2018-01-31 18:01:17 +00:00
definition Loop (G : [n+1;k]GType) : [n;k+1]GType :=
GType.mk (ptrunctype.mk (Ω G) !is_trunc_loop_nat pt)
2018-01-19 15:07:28 +00:00
(connconnect k (B G))
(loop_pequiv_loop (e G) ⬝e* (loopn_connect k (B G))⁻¹ᵉ*)
2018-01-31 18:01:17 +00:00
definition Deloop_adjoint_Loop (G : [n;k+1]GType) (H : [n+1;k]GType) :
2018-01-19 15:07:28 +00:00
ppmap (B (Deloop G)) (B H) ≃* ppmap (B G) (B (Loop H)) :=
(connect_intro_pequiv _ !is_conn_pconntype)⁻¹ᵉ*
2018-01-19 15:07:28 +00:00
2018-01-31 18:01:17 +00:00
definition Deloop_adjoint_Loop_natural {G G' : [n;k+1]GType} {H H' : [n+1;k]GType}
(g : B G' →* B G) (h : B H →* B H') :
psquare (Deloop_adjoint_Loop G H)
(Deloop_adjoint_Loop G' H')
(ppcompose_left h ∘* ppcompose_right g)
(ppcompose_left (connect_functor k h) ∘* ppcompose_right g) :=
(connect_intro_pequiv_natural g h _ _)⁻¹ʰ*
2018-01-31 18:01:17 +00:00
definition Loop_Deloop (G : [n;k+1]GType) : Loop (Deloop G) = G :=
GType_eq (connect_pequiv (is_conn_pconntype (B G)))
2018-01-19 15:07:28 +00:00
2018-01-31 18:01:17 +00:00
definition Forget (G : [n;k+1]GType) : [n;k]GType :=
2018-01-18 19:50:26 +00:00
have is_conn k (B G), from !is_conn_pconntype,
2018-01-31 18:01:17 +00:00
GType.mk G (pconntype.mk (Ω (B G)) !is_conn_loop pt)
2018-01-18 19:50:26 +00:00
abstract begin
refine e G ⬝e* !loopn_succ_in
end end
2018-01-31 18:01:17 +00:00
definition Stabilize (G : [n;k]GType) : [n;k+1]GType :=
2018-01-18 19:50:26 +00:00
have is_conn k (susp (B G)), from !is_conn_susp,
have Hconn : is_conn k (ptrunc (n + k + 1) (susp (B G))), from !is_conn_ptrunc,
2018-01-31 18:01:17 +00:00
GType.mk (ptrunctype.mk (ptrunc n (Ω[k+1] (susp (B G)))) _ pt)
2018-01-18 19:50:26 +00:00
(pconntype.mk (ptrunc (n+k+1) (susp (B G))) Hconn pt)
abstract begin
refine !loopn_ptrunc_pequiv⁻¹ᵉ* ⬝e* _,
apply loopn_pequiv_loopn,
exact ptrunc_change_index !of_nat_add_of_nat _
end end
2018-02-01 02:39:01 +00:00
definition Stabilize_pequiv {G H : [n;k]GType} (e : B G ≃* B H) :
B (Stabilize G) ≃* B (Stabilize H) :=
ptrunc_pequiv_ptrunc (n+k+1) (susp_pequiv e)
2018-01-31 18:01:17 +00:00
definition Stabilize_adjoint_Forget (G : [n;k]GType) (H : [n;k+1]GType) :
2018-01-30 21:11:13 +00:00
ppmap (B (Stabilize G)) (B H) ≃* ppmap (B G) (B (Forget H)) :=
have is_trunc (n + k + 1) (B H), from !is_trunc_B,
pmap_ptrunc_pequiv (n + k + 1) (⅀ (B G)) (B H) ⬝e* susp_adjoint_loop (B G) (B H)
2018-01-31 18:01:17 +00:00
definition Stabilize_adjoint_Forget_natural {G G' : [n;k]GType} {H H' : [n;k+1]GType}
(g : B G' →* B G) (h : B H →* B H') :
psquare (Stabilize_adjoint_Forget G H)
(Stabilize_adjoint_Forget G' H')
(ppcompose_left h ∘* ppcompose_right (ptrunc_functor (n+k+1) (⅀→ g)))
(ppcompose_left (Ω→ h) ∘* ppcompose_right g) :=
begin
have is_trunc (n + k + 1) (B H), from !is_trunc_B,
have is_trunc (n + k + 1) (B H'), from !is_trunc_B,
refine pmap_ptrunc_pequiv_natural (n+k+1) (⅀→ g) h ⬝h* _,
exact susp_adjoint_loop_natural_left g ⬝v* susp_adjoint_loop_natural_right h
end
2018-01-31 18:01:17 +00:00
definition Forget_Stabilize (H : k ≥ n + 2) (G : [n;k]GType) : B (Forget (Stabilize G)) ≃* B G :=
loop_ptrunc_pequiv _ _ ⬝e*
begin
cases k with k,
{ cases H },
{ have k ≥ succ n, from le_of_succ_le_succ H,
assert this : n + succ k ≤ 2 * k,
{ rewrite [two_mul, add_succ, -succ_add], exact nat.add_le_add_right this k },
2018-09-07 14:30:39 +00:00
exact freudenthal_pequiv this (B G) }
end⁻¹ᵉ* ⬝e*
ptrunc_pequiv (n + k) _
2018-01-31 18:01:17 +00:00
definition Stabilize_Forget (H : k ≥ n + 1) (G : [n;k+1]GType) : B (Stabilize (Forget G)) ≃* B G :=
begin
assert lem1 : n + succ k ≤ 2 * k,
{ rewrite [two_mul, add_succ, -succ_add], exact nat.add_le_add_right H k },
have is_conn k (B G), from !is_conn_pconntype,
2018-01-31 18:01:17 +00:00
have Π(G' : [n;k+1]GType), is_trunc (n + k + 1) (B G'), from is_trunc_B,
note z := is_conn_fun_loop_susp_counit (B G) (nat.le_refl (2 * k)),
refine ptrunc_pequiv_ptrunc_of_le (of_nat_le_of_nat lem1) (@(ptrunc_pequiv_ptrunc_of_is_conn_fun _ _) z) ⬝e*
!ptrunc_pequiv,
end
2018-01-19 15:07:28 +00:00
2018-01-30 21:11:13 +00:00
definition stabilization (H : k ≥ n + 2) : is_equiv (@Stabilize n k) :=
begin
fapply adjointify,
{ exact Forget },
2018-01-31 18:01:17 +00:00
{ intro G, apply GType_eq, exact Stabilize_Forget (le.trans !self_le_succ H) _ },
{ intro G, apply GType_eq, exact Forget_Stabilize H G }
end
2018-01-18 19:50:26 +00:00
2018-02-01 02:39:01 +00:00
/- an incomplete formalization of ω-Stabilization -/
definition ωForget (k : ) (G : [n;ω]GType) : [n;k]GType :=
have is_trunc (n + k) (oB G k), from _,
have is_trunc n (Ω[k] (oB G k)), from !is_trunc_loopn_nat,
GType.mk (ptrunctype.mk (Ω[k] (oB G k)) _ pt) (oB G k) (pequiv_of_equiv erfl idp)
definition nStabilize (H : k ≤ l) (G : GType.{u} n k) : GType.{u} n l :=
2018-01-30 21:11:13 +00:00
begin
2018-02-01 02:39:01 +00:00
induction H with l H IH, exact G, exact Stabilize IH
2018-01-30 21:11:13 +00:00
end
2018-01-18 19:50:26 +00:00
2018-02-01 02:39:01 +00:00
definition nStabilize_pequiv (H H' : k ≤ l) {G G' : [n;k]GType}
(e : B G ≃* B G') : B (nStabilize H G) ≃* B (nStabilize H' G') :=
begin
induction H with l H IH,
{ exact e ⬝e* pequiv_ap (λH, B (nStabilize H G')) (is_prop.elim (le.refl k) H') },
cases H' with l H'',
{ exfalso, exact not_succ_le_self H },
exact Stabilize_pequiv (IH H'')
end
definition nStabilize_pequiv_of_eq (H : k ≤ l) (p : k = l) (G : [n;k]GType) :
B (nStabilize H G) ≃* B G :=
begin induction p, exact pequiv_ap (λH, B (nStabilize H G)) (is_prop.elim H (le.refl k)) end
2018-01-18 19:50:26 +00:00
2018-01-31 18:01:17 +00:00
definition ωStabilize_of_le (H : k ≥ n + 2) (G : [n;k]GType) : [n;ω]GType :=
ωGType.mk_le k (λl H', GType_equiv n l (nStabilize H' G))
2018-02-01 02:39:01 +00:00
(λl H', (Forget_Stabilize (le.trans H H') (nStabilize H' G))⁻¹ᵉ*)
definition ωStabilize_of_le_beta (H : k ≥ n + 2) (G : [n;k]GType) (H' : l ≥ k) :
oB (ωStabilize_of_le H G) l ≃* GType_equiv n l (nStabilize H' G) :=
ptruncconntype_eq_equiv _ _ !rec_down_le_beta_ge
definition ωStabilize_of_le_pequiv (H : k ≥ n + 2) (H' : k' ≥ n + 2) {G : [n;k]GType}
{G' : [n;k']GType} (e : B G ≃* B G') (l : ) (Hl : l ≥ k) (Hl' : l ≥ k') (p : k = k') :
oB (ωStabilize_of_le H G) l ≃* oB (ωStabilize_of_le H' G') l :=
begin
refine ωStabilize_of_le_beta H G Hl ⬝e* _ ⬝e* (ωStabilize_of_le_beta H' G' Hl')⁻¹ᵉ*,
induction p,
exact nStabilize_pequiv _ _ e
end
definition ωForget_ωStabilize_of_le (H : k ≥ n + 2) (G : [n;k]GType) :
B (ωForget k (ωStabilize_of_le H G)) ≃* B G :=
ωStabilize_of_le_beta H _ (le.refl k)
2018-01-19 15:07:28 +00:00
2018-01-31 18:01:17 +00:00
definition ωStabilize (G : [n;k]GType) : [n;ω]GType :=
2018-01-18 19:50:26 +00:00
ωStabilize_of_le !le_max_left (nStabilize !le_max_right G)
2018-02-01 02:39:01 +00:00
definition ωForget_ωStabilize (H : k ≥ n + 2) (G : [n;k]GType) :
B (ωForget k (ωStabilize G)) ≃* B G :=
begin
refine _ ⬝e* ωForget_ωStabilize_of_le H G,
esimp [ωForget, ωStabilize],
have H' : max (n + 2) k = k, from max_eq_right H,
exact ωStabilize_of_le_pequiv !le_max_left H (nStabilize_pequiv_of_eq _ H'⁻¹ _)
k (le_of_eq H') (le.refl k) H'
end
/-
definition ωStabilize_adjoint_ωForget (G : [n;k]GType) (H : [n;ω]GType) :
ωGType_hom (ωStabilize G) H ≃* ppmap (B G) (B (ωForget k H)) :=
sorry
2018-02-01 02:39:01 +00:00
definition ωStabilize_ωForget (G : [n;ω]GType) (l : ) :
oB (ωStabilize (ωForget k G)) l ≃* oB G l :=
begin
exact sorry
end
2018-02-01 02:39:01 +00:00
definition ωstabilization (H : k ≥ n + 2) : is_equiv (@ωStabilize n k) :=
begin
apply adjointify _ (ωForget k),
{ intro G', exact sorry },
{ intro G, apply GType_eq, exact ωForget_ωStabilize H G }
end
-/
2018-01-31 18:01:17 +00:00
definition is_trunc_GType_hom (G H : [n;k]GType) : is_trunc n (GType_hom G H) :=
is_trunc_pmap_of_is_conn _ (k.-2) _ _ (k + n) _ (le_of_eq (sub_one_add_plus_two_sub_one k n)⁻¹)
(is_trunc_B' H)
2018-01-31 18:01:17 +00:00
definition is_set_GType_hom (G H : [0;k]GType) : is_set (GType_hom G H) :=
is_trunc_GType_hom G H
2018-01-31 18:01:17 +00:00
definition is_trunc_GType (n k : ) : is_trunc (n + 1) [n;k]GType :=
2018-01-21 11:28:43 +00:00
begin
2018-01-31 18:01:17 +00:00
apply @is_trunc_equiv_closed_rev _ _ (n + 1) (GType_equiv n k),
2018-01-21 11:28:43 +00:00
apply is_trunc_succ_intro, intros X Y,
apply @is_trunc_equiv_closed_rev _ _ _ (ptruncconntype_eq_equiv X Y),
apply @is_trunc_equiv_closed_rev _ _ _ (pequiv.sigma_char_pmap X Y),
2018-01-21 11:28:43 +00:00
apply @is_trunc_subtype (X →* Y) (λ f, trunctype.mk' -1 (is_equiv f)),
2018-01-31 18:01:17 +00:00
exact is_trunc_GType_hom ((GType_equiv n k)⁻¹ᵉ X) ((GType_equiv n k)⁻¹ᵉ Y)
2018-01-21 11:28:43 +00:00
end
2018-01-31 18:01:17 +00:00
local attribute [instance] is_set_GType_hom
2018-01-31 18:01:17 +00:00
definition cGType [constructor] (k : ) : Precategory :=
pb_Precategory (cptruncconntype' (k.-1))
2018-02-01 02:39:01 +00:00
(GType_equiv 0 k ⬝e ptruncconntype_equiv (ap of_nat (zero_add k)) idp ⬝e
(ptruncconntype'_equiv_ptruncconntype (k.-1))⁻¹ᵉ)
2018-01-31 18:01:17 +00:00
example (k : ) : Precategory.carrier (cGType k) = [0;k]GType := by reflexivity
2018-02-01 02:39:01 +00:00
example (k : ) (G H : cGType k) : (G ⟶ H) = (B G →* B H) := by reflexivity
2018-01-31 18:01:17 +00:00
definition cGType_equivalence_cType [constructor] (k : ) : cGType k ≃c cType*[k.-1] :=
!pb_Precategory_equivalence_of_equiv
2018-01-31 18:01:17 +00:00
definition cGType_equivalence_Grp [constructor] : cGType.{u} 1 ≃c Grp.{u} :=
equivalence.trans !pb_Precategory_equivalence_of_equiv
(equivalence.trans (equivalence.symm Grp_equivalence_cptruncconntype')
proof equivalence.refl _ qed)
2018-01-31 18:01:17 +00:00
definition cGType_equivalence_AbGrp [constructor] (k : ) : cGType.{u} (k+2) ≃c AbGrp.{u} :=
equivalence.trans !pb_Precategory_equivalence_of_equiv
(equivalence.trans (equivalence.symm (AbGrp_equivalence_cptruncconntype' k))
proof equivalence.refl _ qed)
2018-09-07 14:30:39 +00:00
/-
2018-02-01 02:39:01 +00:00
print axioms GType_equiv
print axioms InfGType_equiv
print axioms Decat_adjoint_Disc
print axioms Decat_adjoint_Disc_natural
2018-02-01 02:39:01 +00:00
print axioms InfDecat_adjoint_InfDisc
print axioms InfDecat_adjoint_InfDisc_natural
print axioms Deloop_adjoint_Loop
print axioms Deloop_adjoint_Loop_natural
2018-01-30 21:11:13 +00:00
print axioms Stabilize_adjoint_Forget
print axioms Stabilize_adjoint_Forget_natural
print axioms stabilization
2018-01-31 18:01:17 +00:00
print axioms is_trunc_GType
print axioms cGType_equivalence_Grp
print axioms cGType_equivalence_AbGrp
2018-09-07 14:30:39 +00:00
-/
end higher_group