mathlib3 documentation

topology.homotopy.H_spaces

H-spaces #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This file defines H-spaces mainly following the approach proposed by Serre in his paper Homologie singulière des espaces fibrés. The idea beaneath H-spaces is that they are topological spaces with a binary operation ⋀ : X → X → X that is a homotopic-theoretic weakening of an operation what would make X into a topological monoid. In particular, there exists a "neutral element" e : X such that λ x, e ⋀ x and λ x, x ⋀ e are homotopic to the identity on X, see the Wikipedia page of H-spaces.

Some notable properties of H-spaces are

Main Results #

To Do #

References #

@[class]
structure H_space (X : Type u) [topological_space X] :

A topological space X is an H-space if it behaves like a (potentially non-associative) topological group, but where the axioms for a group only hold up to homotopy.

Instances of this typeclass
Instances of other typeclasses for H_space
  • H_space.has_sizeof_inst
@[protected, instance]
def H_space.prod (X : Type u) (Y : Type v) [topological_space X] [topological_space Y] [H_space X] [H_space Y] :
H_space (X × Y)
Equations

The definition to_H_space is not an instance because its @additive version would lead to a diamond since a topological field would inherit two H_space structures, one from the mul_one_class and one from the add_zero_class. In the case of a group, we make topological_group.H_space an instance."

Equations

The definition to_H_space is not an instance because it comes together with a multiplicative version which would lead to a diamond since a topological field would inherit two H_space structures, one from the mul_one_class and one from the add_zero_class. In the case of an additive group, we make topological_group.H_space an instance.

Equations

Q_right is analogous to the function Q defined on p. 475 of [Ser51] that helps proving continuity of delay_refl_right.

Equations
noncomputable def path.delay_refl_right {X : Type u} [topological_space X] {x y : X} (θ : unit_interval) (γ : path x y) :
path x y

This is the function analogous to the one on p. 475 of [Ser51], defining a homotopy from the product path γ ∧ e to γ.

Equations
theorem path.delay_refl_right_zero {X : Type u} [topological_space X] {x y : X} (γ : path x y) :
theorem path.delay_refl_right_one {X : Type u} [topological_space X] {x y : X} (γ : path x y) :
noncomputable def path.delay_refl_left {X : Type u} [topological_space X] {x y : X} (θ : unit_interval) (γ : path x y) :
path x y

This is the function on p. 475 of [Ser51], defining a homotopy from a path γ to the product path e ∧ γ.

Equations
theorem path.delay_refl_left_zero {X : Type u} [topological_space X] {x y : X} (γ : path x y) :
theorem path.delay_refl_left_one {X : Type u} [topological_space X] {x y : X} (γ : path x y) :
@[protected, instance]
noncomputable def path.H_space {X : Type u} [topological_space X] (x : X) :

The loop space at x carries a structure of a H-space. Note that the field e_Hmul (resp. Hmul_e) neither implies nor is implied by path.homotopy.refl_trans (resp. path.homotopy.trans_refl).

Equations