Homotopy equivalences between topological spaces #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file, we define homotopy equivalences between topological spaces X and Y as a pair of
functions f : C(X, Y) and g : C(Y, X) such that f.comp g and g.comp f are both homotopic
to id.
Main definitions #
continuous_map.homotopy_equivis the type of homotopy equivalences between topological spaces.
Notation #
We introduce the notation X ≃ₕ Y for continuous_map.homotopy_equiv X Y in the continuous_map
locale.
- to_fun : C(X, Y)
- inv_fun : C(Y, X)
- left_inv : (self.inv_fun.comp self.to_fun).homotopic (continuous_map.id X)
- right_inv : (self.to_fun.comp self.inv_fun).homotopic (continuous_map.id Y)
A homotopy equivalence between topological spaces X and Y are a pair of functions
to_fun : C(X, Y) and inv_fun : C(Y, X) such that to_fun.comp inv_fun and inv_fun.comp to_fun
are both homotopic to id.
Instances for continuous_map.homotopy_equiv
- continuous_map.homotopy_equiv.has_sizeof_inst
- continuous_map.homotopy_equiv.has_coe_to_fun
- continuous_map.homotopy_equiv.inhabited
Equations
- continuous_map.homotopy_equiv.has_coe_to_fun = {coe := λ (h : continuous_map.homotopy_equiv X Y), ⇑(h.to_fun)}
Any homeomorphism is a homotopy equivalence.
If X is homotopy equivalent to Y, then Y is homotopy equivalent to X.
See Note [custom simps projection]. We need to specify this projection explicitly in this case, because it is a composition of multiple projections.
Equations
See Note [custom simps projection]. We need to specify this projection explicitly in this case, because it is a composition of multiple projections.
Equations
Any topological space is homotopy equivalent to itself.
Equations
If X is homotopy equivalent to Y, and Y is homotopy equivalent to Z, then X is homotopy
equivalent to Z.