2015-09-13 18:58:11 +00:00
|
|
|
|
/-
|
|
|
|
|
Copyright (c) 2015 Ulrik Buchholtz. All rights reserved.
|
|
|
|
|
Released under Apache 2.0 license as described in the file LICENSE.
|
2016-02-26 22:00:28 +00:00
|
|
|
|
Authors: Ulrik Buchholtz, Floris van Doorn
|
2015-09-13 18:58:11 +00:00
|
|
|
|
-/
|
2016-03-02 21:23:24 +00:00
|
|
|
|
import types.trunc types.arrow_2 .sphere
|
2015-09-13 18:58:11 +00:00
|
|
|
|
|
2016-02-26 22:00:28 +00:00
|
|
|
|
open eq is_trunc is_equiv nat equiv trunc function fiber funext pi
|
2015-09-13 18:58:11 +00:00
|
|
|
|
|
|
|
|
|
namespace homotopy
|
|
|
|
|
|
2016-02-26 22:00:28 +00:00
|
|
|
|
definition is_conn [reducible] (n : ℕ₋₂) (A : Type) : Type :=
|
2015-09-13 18:58:11 +00:00
|
|
|
|
is_contr (trunc n A)
|
|
|
|
|
|
2016-02-26 22:00:28 +00:00
|
|
|
|
definition is_conn_equiv_closed (n : ℕ₋₂) {A B : Type}
|
2015-11-05 19:37:46 +00:00
|
|
|
|
: A ≃ B → is_conn n A → is_conn n B :=
|
|
|
|
|
begin
|
|
|
|
|
intros H C,
|
|
|
|
|
fapply @is_contr_equiv_closed (trunc n A) _,
|
|
|
|
|
apply trunc_equiv_trunc,
|
|
|
|
|
assumption
|
|
|
|
|
end
|
|
|
|
|
|
2016-03-06 16:24:59 +00:00
|
|
|
|
definition is_conn_fun [reducible] (n : ℕ₋₂) {A B : Type} (f : A → B) : Type :=
|
2015-09-13 18:58:11 +00:00
|
|
|
|
Πb : B, is_conn n (fiber f b)
|
|
|
|
|
|
2016-03-06 00:35:12 +00:00
|
|
|
|
theorem is_conn_of_le (A : Type) {n k : ℕ₋₂} (H : n ≤ k) [is_conn k A] : is_conn n A :=
|
|
|
|
|
begin
|
|
|
|
|
apply is_contr_equiv_closed,
|
|
|
|
|
apply trunc_trunc_equiv_left _ n k H
|
|
|
|
|
end
|
|
|
|
|
|
2016-03-06 16:24:59 +00:00
|
|
|
|
theorem is_conn_fun_of_le {A B : Type} (f : A → B) {n k : ℕ₋₂} (H : n ≤ k)
|
|
|
|
|
[is_conn_fun k f] : is_conn_fun n f :=
|
2016-03-06 00:35:12 +00:00
|
|
|
|
λb, is_conn_of_le _ H
|
|
|
|
|
|
2016-03-06 16:24:59 +00:00
|
|
|
|
namespace is_conn_fun
|
2015-11-05 19:37:46 +00:00
|
|
|
|
section
|
2016-03-06 16:24:59 +00:00
|
|
|
|
parameters (n : ℕ₋₂) {A B : Type} {h : A → B}
|
|
|
|
|
(H : is_conn_fun n h) (P : B → Type) [Πb, is_trunc n (P b)]
|
2015-11-05 19:37:46 +00:00
|
|
|
|
|
2016-01-23 19:15:59 +00:00
|
|
|
|
private definition rec.helper : (Πa : A, P (h a)) → Πb : B, trunc n (fiber h b) → P b :=
|
2015-11-05 19:37:46 +00:00
|
|
|
|
λt b, trunc.rec (λx, point_eq x ▸ t (point x))
|
|
|
|
|
|
2016-01-23 19:15:59 +00:00
|
|
|
|
private definition rec.g : (Πa : A, P (h a)) → (Πb : B, P b) :=
|
|
|
|
|
λt b, rec.helper t b (@center (trunc n (fiber h b)) (H b))
|
2015-11-05 19:37:46 +00:00
|
|
|
|
|
|
|
|
|
-- induction principle for n-connected maps (Lemma 7.5.7)
|
2016-01-23 19:15:59 +00:00
|
|
|
|
protected definition rec : is_equiv (λs : Πb : B, P b, λa : A, s (h a)) :=
|
|
|
|
|
adjointify (λs a, s (h a)) rec.g
|
2015-11-05 19:37:46 +00:00
|
|
|
|
begin
|
2016-01-23 19:15:59 +00:00
|
|
|
|
intro t, apply eq_of_homotopy, intro a, unfold rec.g, unfold rec.helper,
|
2015-11-05 19:37:46 +00:00
|
|
|
|
rewrite [@center_eq _ (H (h a)) (tr (fiber.mk a idp))],
|
|
|
|
|
end
|
|
|
|
|
begin
|
2016-01-23 19:15:59 +00:00
|
|
|
|
intro k, apply eq_of_homotopy, intro b, unfold rec.g,
|
2015-11-05 19:37:46 +00:00
|
|
|
|
generalize (@center _ (H b)), apply trunc.rec, apply fiber.rec,
|
|
|
|
|
intros a p, induction p, reflexivity
|
|
|
|
|
end
|
|
|
|
|
|
2016-01-23 19:15:59 +00:00
|
|
|
|
protected definition elim : (Πa : A, P (h a)) → (Πb : B, P b) :=
|
2015-11-05 19:37:46 +00:00
|
|
|
|
@is_equiv.inv _ _ (λs a, s (h a)) rec
|
|
|
|
|
|
2016-01-23 19:15:59 +00:00
|
|
|
|
protected definition elim_β : Πf : (Πa : A, P (h a)), Πa : A, elim f (h a) = f a :=
|
2015-11-05 19:37:46 +00:00
|
|
|
|
λf, apd10 (@is_equiv.right_inv _ _ (λs a, s (h a)) rec f)
|
|
|
|
|
|
|
|
|
|
end
|
|
|
|
|
|
2016-01-23 19:15:59 +00:00
|
|
|
|
section
|
2016-03-06 16:24:59 +00:00
|
|
|
|
parameters (n k : ℕ₋₂) {A B : Type} {f : A → B}
|
|
|
|
|
(H : is_conn_fun n f) (P : B → Type) [HP : Πb, is_trunc (n +2+ k) (P b)]
|
2016-01-23 19:15:59 +00:00
|
|
|
|
|
2016-03-06 16:24:59 +00:00
|
|
|
|
include H HP
|
2016-01-23 19:15:59 +00:00
|
|
|
|
-- Lemma 8.6.1
|
2016-02-26 22:00:28 +00:00
|
|
|
|
proposition elim_general : is_trunc_fun k (pi_functor_left f P) :=
|
2016-01-23 19:15:59 +00:00
|
|
|
|
begin
|
2016-03-06 16:24:59 +00:00
|
|
|
|
revert P HP,
|
|
|
|
|
induction k with k IH: intro P HP t,
|
|
|
|
|
{ apply is_contr_fiber_of_is_equiv, apply is_conn_fun.rec, exact H, exact HP},
|
2016-01-23 19:15:59 +00:00
|
|
|
|
{ apply is_trunc_succ_intro,
|
|
|
|
|
intros x y, cases x with g p, cases y with h q,
|
2016-02-29 20:11:17 +00:00
|
|
|
|
have e : fiber (λr : g ~ h, (λa, r (f a))) (apd10 (p ⬝ q⁻¹))
|
2016-01-23 19:15:59 +00:00
|
|
|
|
≃ (fiber.mk g p = fiber.mk h q
|
|
|
|
|
:> fiber (λs : (Πb, P b), (λa, s (f a))) t),
|
2016-02-29 20:11:17 +00:00
|
|
|
|
begin
|
|
|
|
|
apply equiv.trans !fiber.sigma_char,
|
|
|
|
|
have e' : Πr : g ~ h,
|
2016-01-23 19:15:59 +00:00
|
|
|
|
((λa, r (f a)) = apd10 (p ⬝ q⁻¹))
|
|
|
|
|
≃ (ap (λv, (λa, v (f a))) (eq_of_homotopy r) ⬝ q = p),
|
2016-02-29 20:11:17 +00:00
|
|
|
|
begin
|
|
|
|
|
intro r,
|
2016-01-23 19:15:59 +00:00
|
|
|
|
refine equiv.trans _ (eq_con_inv_equiv_con_eq q p
|
|
|
|
|
(ap (λv a, v (f a)) (eq_of_homotopy r))),
|
|
|
|
|
rewrite [-(ap (λv a, v (f a)) (apd10_eq_of_homotopy r))],
|
|
|
|
|
rewrite [-(apd10_ap_precompose_dependent f (eq_of_homotopy r))],
|
|
|
|
|
apply equiv.symm,
|
2016-02-29 20:11:17 +00:00
|
|
|
|
apply eq_equiv_fn_eq (@apd10 A (λa, P (f a)) (λa, g (f a)) (λa, h (f a)))
|
|
|
|
|
end,
|
2016-02-15 21:05:31 +00:00
|
|
|
|
apply equiv.trans (sigma.sigma_equiv_sigma_right e'), clear e',
|
2016-01-23 19:15:59 +00:00
|
|
|
|
apply equiv.trans (equiv.symm (sigma.sigma_equiv_sigma_left
|
|
|
|
|
eq_equiv_homotopy)),
|
|
|
|
|
apply equiv.symm, apply equiv.trans !fiber_eq_equiv,
|
2016-02-15 21:05:31 +00:00
|
|
|
|
apply sigma.sigma_equiv_sigma_right, intro r,
|
2016-02-29 20:11:17 +00:00
|
|
|
|
apply eq_equiv_eq_symm
|
|
|
|
|
end,
|
2016-01-23 19:15:59 +00:00
|
|
|
|
apply @is_trunc_equiv_closed _ _ k e, clear e,
|
2016-03-06 16:24:59 +00:00
|
|
|
|
apply IH (λb : B, (g b = h b)) (λb, @is_trunc_eq (P b) (n +2+ k) (HP b) (g b) (h b))}
|
2016-01-23 19:15:59 +00:00
|
|
|
|
end
|
2016-02-26 22:00:28 +00:00
|
|
|
|
|
2016-01-23 19:15:59 +00:00
|
|
|
|
end
|
|
|
|
|
|
2015-11-05 19:37:46 +00:00
|
|
|
|
section
|
|
|
|
|
universe variables u v
|
2016-03-06 16:24:59 +00:00
|
|
|
|
parameters (n : ℕ₋₂) {A : Type.{u}} {B : Type.{v}} {h : A → B}
|
2015-11-05 19:37:46 +00:00
|
|
|
|
parameter sec : ΠP : B → trunctype.{max u v} n,
|
|
|
|
|
is_retraction (λs : (Πb : B, P b), λ a, s (h a))
|
|
|
|
|
|
|
|
|
|
private definition s := sec (λb, trunctype.mk' n (trunc n (fiber h b)))
|
|
|
|
|
|
|
|
|
|
include sec
|
|
|
|
|
|
|
|
|
|
-- the other half of Lemma 7.5.7
|
2016-03-06 16:24:59 +00:00
|
|
|
|
definition intro : is_conn_fun n h :=
|
2015-11-05 19:37:46 +00:00
|
|
|
|
begin
|
|
|
|
|
intro b,
|
|
|
|
|
apply is_contr.mk (@is_retraction.sect _ _ _ s (λa, tr (fiber.mk a idp)) b),
|
2016-02-16 01:59:38 +00:00
|
|
|
|
esimp, apply trunc.rec, apply fiber.rec, intros a p,
|
2015-11-05 19:37:46 +00:00
|
|
|
|
apply transport
|
|
|
|
|
(λz : (Σy, h a = y), @sect _ _ _ s (λa, tr (mk a idp)) (sigma.pr1 z) =
|
|
|
|
|
tr (fiber.mk a (sigma.pr2 z)))
|
|
|
|
|
(@center_eq _ (is_contr_sigma_eq (h a)) (sigma.mk b p)),
|
|
|
|
|
exact apd10 (@right_inverse _ _ _ s (λa, tr (fiber.mk a idp))) a
|
|
|
|
|
end
|
|
|
|
|
end
|
2016-03-06 16:24:59 +00:00
|
|
|
|
end is_conn_fun
|
2015-11-05 19:37:46 +00:00
|
|
|
|
|
|
|
|
|
-- Connectedness is related to maps to and from the unit type, first to
|
|
|
|
|
section
|
2016-02-26 22:00:28 +00:00
|
|
|
|
parameters (n : ℕ₋₂) (A : Type)
|
2015-11-05 19:37:46 +00:00
|
|
|
|
|
|
|
|
|
definition is_conn_of_map_to_unit
|
2016-03-06 16:24:59 +00:00
|
|
|
|
: is_conn_fun n (const A unit.star) → is_conn n A :=
|
2015-11-05 19:37:46 +00:00
|
|
|
|
begin
|
2016-03-06 16:24:59 +00:00
|
|
|
|
intro H, unfold is_conn_fun at H,
|
2015-11-05 19:37:46 +00:00
|
|
|
|
rewrite [-(ua (fiber.fiber_star_equiv A))],
|
|
|
|
|
exact (H unit.star)
|
|
|
|
|
end
|
|
|
|
|
|
|
|
|
|
-- now maps from unit
|
2016-03-06 16:24:59 +00:00
|
|
|
|
definition is_conn_of_map_from_unit (a₀ : A) (H : is_conn_fun n (const unit a₀))
|
2015-11-05 19:37:46 +00:00
|
|
|
|
: is_conn n .+1 A :=
|
|
|
|
|
is_contr.mk (tr a₀)
|
|
|
|
|
begin
|
|
|
|
|
apply trunc.rec, intro a,
|
|
|
|
|
exact trunc.elim (λz : fiber (const unit a₀) a, ap tr (point_eq z))
|
|
|
|
|
(@center _ (H a))
|
|
|
|
|
end
|
|
|
|
|
|
2016-03-06 16:24:59 +00:00
|
|
|
|
definition is_conn_fun_from_unit (a₀ : A) [H : is_conn n .+1 A]
|
|
|
|
|
: is_conn_fun n (const unit a₀) :=
|
2015-11-05 19:37:46 +00:00
|
|
|
|
begin
|
|
|
|
|
intro a,
|
|
|
|
|
apply is_conn_equiv_closed n (equiv.symm (fiber_const_equiv A a₀ a)),
|
|
|
|
|
apply @is_contr_equiv_closed _ _ (tr_eq_tr_equiv n a₀ a),
|
|
|
|
|
end
|
|
|
|
|
|
2015-09-13 18:58:11 +00:00
|
|
|
|
end
|
|
|
|
|
|
2016-01-23 19:15:59 +00:00
|
|
|
|
-- as special case we get elimination principles for pointed connected types
|
|
|
|
|
namespace is_conn
|
2016-02-15 23:23:28 +00:00
|
|
|
|
open pointed unit
|
2016-01-23 19:15:59 +00:00
|
|
|
|
section
|
2016-03-06 16:24:59 +00:00
|
|
|
|
parameters (n : ℕ₋₂) {A : Type*}
|
|
|
|
|
[H : is_conn n .+1 A] (P : A → Type) [Πa, is_trunc n (P a)]
|
2016-01-23 19:15:59 +00:00
|
|
|
|
|
|
|
|
|
include H
|
|
|
|
|
protected definition rec : is_equiv (λs : Πa : A, P a, s (Point A)) :=
|
|
|
|
|
@is_equiv_compose
|
|
|
|
|
(Πa : A, P a) (unit → P (Point A)) (P (Point A))
|
|
|
|
|
(λs x, s (Point A)) (λf, f unit.star)
|
2016-03-06 16:24:59 +00:00
|
|
|
|
(is_conn_fun.rec n (is_conn_fun_from_unit n A (Point A)) P)
|
2016-03-01 04:37:03 +00:00
|
|
|
|
(to_is_equiv (arrow_unit_left (P (Point A))))
|
2016-01-23 19:15:59 +00:00
|
|
|
|
|
|
|
|
|
protected definition elim : P (Point A) → (Πa : A, P a) :=
|
|
|
|
|
@is_equiv.inv _ _ (λs, s (Point A)) rec
|
|
|
|
|
|
|
|
|
|
protected definition elim_β (p : P (Point A)) : elim p (Point A) = p :=
|
|
|
|
|
@is_equiv.right_inv _ _ (λs, s (Point A)) rec p
|
|
|
|
|
end
|
|
|
|
|
|
|
|
|
|
section
|
2016-03-06 16:24:59 +00:00
|
|
|
|
parameters (n k : ℕ₋₂) {A : Type*}
|
|
|
|
|
[H : is_conn n .+1 A] (P : A → Type) [Πa, is_trunc (n +2+ k) (P a)]
|
2016-01-23 19:15:59 +00:00
|
|
|
|
|
|
|
|
|
include H
|
|
|
|
|
proposition elim_general (p : P (Point A))
|
|
|
|
|
: is_trunc k (fiber (λs : (Πa : A, P a), s (Point A)) p) :=
|
|
|
|
|
@is_trunc_equiv_closed
|
|
|
|
|
(fiber (λs x, s (Point A)) (λx, p))
|
|
|
|
|
(fiber (λs, s (Point A)) p)
|
|
|
|
|
k
|
2016-03-01 04:37:03 +00:00
|
|
|
|
(equiv.symm (fiber.equiv_postcompose (to_fun (arrow_unit_left (P (Point A))))))
|
2016-03-06 16:24:59 +00:00
|
|
|
|
(is_conn_fun.elim_general n k (is_conn_fun_from_unit n A (Point A)) P (λx, p))
|
2016-01-23 19:15:59 +00:00
|
|
|
|
end
|
|
|
|
|
end is_conn
|
|
|
|
|
|
2015-09-13 18:58:11 +00:00
|
|
|
|
-- Lemma 7.5.2
|
|
|
|
|
definition minus_one_conn_of_surjective {A B : Type} (f : A → B)
|
2016-03-06 16:24:59 +00:00
|
|
|
|
: is_surjective f → is_conn_fun -1 f :=
|
2015-09-13 18:58:11 +00:00
|
|
|
|
begin
|
|
|
|
|
intro H, intro b,
|
2016-02-15 20:55:29 +00:00
|
|
|
|
exact @is_contr_of_inhabited_prop (∥fiber f b∥) (is_trunc_trunc -1 (fiber f b)) (H b),
|
2015-09-13 18:58:11 +00:00
|
|
|
|
end
|
|
|
|
|
|
|
|
|
|
definition is_surjection_of_minus_one_conn {A B : Type} (f : A → B)
|
2016-03-06 16:24:59 +00:00
|
|
|
|
: is_conn_fun -1 f → is_surjective f :=
|
2015-09-13 18:58:11 +00:00
|
|
|
|
begin
|
|
|
|
|
intro H, intro b,
|
|
|
|
|
exact @center (∥fiber f b∥) (H b),
|
|
|
|
|
end
|
|
|
|
|
|
2015-09-27 17:30:47 +00:00
|
|
|
|
definition merely_of_minus_one_conn {A : Type} : is_conn -1 A → ∥A∥ :=
|
2015-09-13 18:58:11 +00:00
|
|
|
|
λH, @center (∥A∥) H
|
|
|
|
|
|
|
|
|
|
definition minus_one_conn_of_merely {A : Type} : ∥A∥ → is_conn -1 A :=
|
2016-02-15 20:55:29 +00:00
|
|
|
|
@is_contr_of_inhabited_prop (∥A∥) (is_trunc_trunc -1 A)
|
2015-09-13 18:58:11 +00:00
|
|
|
|
|
2015-09-27 17:30:47 +00:00
|
|
|
|
section
|
|
|
|
|
open arrow
|
|
|
|
|
|
|
|
|
|
variables {f g : arrow}
|
|
|
|
|
|
|
|
|
|
-- Lemma 7.5.4
|
|
|
|
|
definition retract_of_conn_is_conn [instance] (r : arrow_hom f g) [H : is_retraction r]
|
2016-03-06 16:24:59 +00:00
|
|
|
|
(n : ℕ₋₂) [K : is_conn_fun n f] : is_conn_fun n g :=
|
2015-09-27 17:30:47 +00:00
|
|
|
|
begin
|
|
|
|
|
intro b, unfold is_conn,
|
|
|
|
|
apply is_contr_retract (trunc_functor n (retraction_on_fiber r b)),
|
|
|
|
|
exact K (on_cod (arrow.is_retraction.sect r) b)
|
|
|
|
|
end
|
|
|
|
|
|
|
|
|
|
end
|
|
|
|
|
|
|
|
|
|
-- Corollary 7.5.5
|
2016-02-26 22:00:28 +00:00
|
|
|
|
definition is_conn_homotopy (n : ℕ₋₂) {A B : Type} {f g : A → B}
|
2016-03-06 16:24:59 +00:00
|
|
|
|
(p : f ~ g) (H : is_conn_fun n f) : is_conn_fun n g :=
|
2016-02-15 20:18:07 +00:00
|
|
|
|
@retract_of_conn_is_conn _ _ (arrow.arrow_hom_of_homotopy p) (arrow.is_retraction_arrow_hom_of_homotopy p) n H
|
2015-09-27 17:30:47 +00:00
|
|
|
|
|
2015-11-05 19:37:46 +00:00
|
|
|
|
-- all types are -2-connected
|
2016-03-06 00:35:12 +00:00
|
|
|
|
definition is_conn_minus_two (A : Type) : is_conn -2 A :=
|
2015-11-05 19:37:46 +00:00
|
|
|
|
_
|
|
|
|
|
|
|
|
|
|
-- Theorem 8.2.1
|
|
|
|
|
open susp
|
|
|
|
|
|
2016-03-02 21:23:24 +00:00
|
|
|
|
theorem is_conn_susp [instance] (n : ℕ₋₂) (A : Type)
|
2015-11-05 19:37:46 +00:00
|
|
|
|
[H : is_conn n A] : is_conn (n .+1) (susp A) :=
|
|
|
|
|
is_contr.mk (tr north)
|
|
|
|
|
begin
|
|
|
|
|
apply trunc.rec,
|
|
|
|
|
fapply susp.rec,
|
|
|
|
|
{ reflexivity },
|
|
|
|
|
{ exact (trunc.rec (λa, ap tr (merid a)) (center (trunc n A))) },
|
|
|
|
|
{ intro a,
|
|
|
|
|
generalize (center (trunc n A)),
|
|
|
|
|
apply trunc.rec,
|
|
|
|
|
intro a',
|
|
|
|
|
apply pathover_of_tr_eq,
|
|
|
|
|
rewrite [transport_eq_Fr,idp_con],
|
|
|
|
|
revert H, induction n with [n, IH],
|
2016-02-15 20:18:07 +00:00
|
|
|
|
{ intro H, apply is_prop.elim },
|
2015-11-05 19:37:46 +00:00
|
|
|
|
{ intros H,
|
|
|
|
|
change ap (@tr n .+2 (susp A)) (merid a) = ap tr (merid a'),
|
|
|
|
|
generalize a',
|
2016-03-06 16:24:59 +00:00
|
|
|
|
apply is_conn_fun.elim n
|
|
|
|
|
(is_conn_fun_from_unit n A a)
|
2015-11-05 19:37:46 +00:00
|
|
|
|
(λx : A, trunctype.mk' n (ap (@tr n .+2 (susp A)) (merid a) = ap tr (merid x))),
|
|
|
|
|
intros,
|
|
|
|
|
change ap (@tr n .+2 (susp A)) (merid a) = ap tr (merid a),
|
|
|
|
|
reflexivity
|
|
|
|
|
}
|
|
|
|
|
}
|
|
|
|
|
end
|
|
|
|
|
|
2016-03-06 00:35:12 +00:00
|
|
|
|
-- Lemma 7.5.14
|
2016-03-06 16:24:59 +00:00
|
|
|
|
theorem is_equiv_trunc_functor_of_is_conn_fun {A B : Type} (n : ℕ₋₂) (f : A → B)
|
|
|
|
|
[H : is_conn_fun n f] : is_equiv (trunc_functor n f) :=
|
2016-03-06 00:35:12 +00:00
|
|
|
|
begin
|
|
|
|
|
fapply adjointify,
|
|
|
|
|
{ intro b, induction b with b, exact trunc_functor n point (center (trunc n (fiber f b)))},
|
|
|
|
|
{ intro b, induction b with b, esimp, generalize center (trunc n (fiber f b)), intro v,
|
|
|
|
|
induction v with v, induction v with a p, esimp, exact ap tr p},
|
|
|
|
|
{ intro a, induction a with a, esimp, rewrite [center_eq (tr (fiber.mk a idp))]}
|
|
|
|
|
end
|
|
|
|
|
|
2016-03-06 16:24:59 +00:00
|
|
|
|
theorem trunc_equiv_trunc_of_is_conn_fun {A B : Type} (n : ℕ₋₂) (f : A → B)
|
|
|
|
|
[H : is_conn_fun n f] : trunc n A ≃ trunc n B :=
|
|
|
|
|
equiv.mk (trunc_functor n f) (is_equiv_trunc_functor_of_is_conn_fun n f)
|
2016-03-06 00:35:12 +00:00
|
|
|
|
|
|
|
|
|
open trunc_index pointed sphere.ops
|
2016-03-03 15:48:27 +00:00
|
|
|
|
-- Corollary 8.2.2
|
2016-03-06 00:35:12 +00:00
|
|
|
|
theorem is_conn_sphere [instance] (n : ℕ₋₁) : is_conn (n..-1) (S n) :=
|
2016-03-02 21:23:24 +00:00
|
|
|
|
begin
|
|
|
|
|
induction n with n IH,
|
2016-03-06 00:35:12 +00:00
|
|
|
|
{ apply is_conn_minus_two},
|
2016-03-02 21:23:24 +00:00
|
|
|
|
{ rewrite [succ_sub_one, sphere.sphere_succ], apply is_conn_susp}
|
|
|
|
|
end
|
|
|
|
|
|
2016-03-06 00:35:12 +00:00
|
|
|
|
section
|
|
|
|
|
open sphere_index
|
|
|
|
|
theorem is_conn_psphere [instance] (n : ℕ) : is_conn (n.-1) (S. n) :=
|
|
|
|
|
transport (λx, is_conn x (sphere n)) (of_nat_sub_one n) (is_conn_sphere n)
|
|
|
|
|
end
|
|
|
|
|
|
2015-09-13 18:58:11 +00:00
|
|
|
|
end homotopy
|