Spectral/homology/sphere.hlean
Floris van Doorn 3367c20f9d make pointed suspension and spheres the default
There is one proof in realprojective which I couldn't quite fix, so for now I left a sorry
2017-07-20 18:03:13 +01:00

36 lines
1.3 KiB
Text
Raw Blame History

This file contains ambiguous Unicode characters

This file contains Unicode characters that might be confused with other characters. If you think that this is intentional, you can safely ignore this warning. Use the Escape button to reveal them.

/-
Copyright (c) 2017 Kuen-Bang Hou (Favonia).
Released under Apache 2.0 license as described in the file LICENSE.
Author: Kuen-Bang Hou (Favonia)
-/
import .basic
open eq pointed group algebra circle sphere nat equiv susp
function sphere homology int lift
namespace homology
section
parameter (theory : homology_theory)
open homology_theory
theorem Hsphere : Π(n : )(m : ), HH theory n (plift (sphere m)) ≃g HH theory (n - m) (plift (sphere 0)) :=
begin
intros n m, revert n, induction m with m,
{ exact λ n, isomorphism_ap (λ n, HH theory n (plift (sphere 0))) (sub_zero n)⁻¹ },
{ intro n, exact calc
HH theory n (plift (susp (sphere m)))
≃g HH theory (succ (pred n)) (plift (susp (sphere m)))
: by exact isomorphism_ap (λ n, HH theory n (plift (susp (sphere m)))) (succ_pred n)⁻¹
... ≃g HH theory (pred n) (plift (sphere m)) : by exact Hplift_susp theory (pred n) (sphere m)
... ≃g HH theory (pred n - m) (plift (sphere 0)) : by exact v_0 (pred n)
... ≃g HH theory (n - succ m) (plift (sphere 0))
: by exact isomorphism_ap (λ n, HH theory n (plift (sphere 0))) (sub_sub n 1 m ⬝ ap (λ m, n - m) (add.comm 1 m))
}
end
end
end homology