Homeomorphisms #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines homeomorphisms between two topological spaces. They are bijections with both
directions continuous. We denote homeomorphisms with the notation ≃ₜ
.
Main definitions #
homeomorph α β
: The type of homeomorphisms fromα
toβ
. This type can be denoted using the following notation:α ≃ₜ β
.
Main results #
- Pretty much every topological property is preserved under homeomorphisms.
homeomorph.homeomorph_of_continuous_open
: A continuous bijection that is an open map is a homeomorphism.
- to_equiv : α ≃ β
- continuous_to_fun : continuous self.to_equiv.to_fun . "continuity'"
- continuous_inv_fun : continuous self.to_equiv.inv_fun . "continuity'"
Homeomorphism between α
and β
, also called topological isomorphism
Instances for homeomorph
- homeomorph.has_sizeof_inst
- homeomorph.has_coe_to_fun
- homeomorph.continuous_map.has_coe
Inverse of a homeomorphism.
Equations
- h.symm = {to_equiv := h.to_equiv.symm, continuous_to_fun := _, continuous_inv_fun := _}
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]
Equations
Identity map as a homeomorphism.
Equations
- homeomorph.refl α = {to_equiv := equiv.refl α, continuous_to_fun := _, continuous_inv_fun := _}
Composition of two homeomorphisms.
Equations
- h₁.trans h₂ = {to_equiv := h₁.to_equiv.trans h₂.to_equiv, continuous_to_fun := _, continuous_inv_fun := _}
Change the homeomorphism f
to make the inverse function definitionally equal to g
.
Equations
- f.change_inv g hg = have this : g = ⇑(f.symm), from _, {to_equiv := {to_fun := ⇑f, inv_fun := g, left_inv := _, right_inv := _}, continuous_to_fun := _, continuous_inv_fun := _}
Homeomorphism given an embedding.
Equations
- homeomorph.of_embedding f hf = {to_equiv := equiv.of_injective f _, continuous_to_fun := _, continuous_inv_fun := _}
If an bijective map e : α ≃ β
is continuous and open, then it is a homeomorphism.
Equations
- homeomorph.homeomorph_of_continuous_open e h₁ h₂ = {to_equiv := e, continuous_to_fun := h₁, continuous_inv_fun := _}
If two sets are equal, then they are homeomorphic.
Equations
- homeomorph.set_congr h = {to_equiv := equiv.set_congr h, continuous_to_fun := _, continuous_inv_fun := _}
Sum of two homeomorphisms.
Equations
- h₁.sum_congr h₂ = {to_equiv := h₁.to_equiv.sum_congr h₂.to_equiv, continuous_to_fun := _, continuous_inv_fun := _}
Product of two homeomorphisms.
Equations
- h₁.prod_congr h₂ = {to_equiv := h₁.to_equiv.prod_congr h₂.to_equiv, continuous_to_fun := _, continuous_inv_fun := _}
α × β
is homeomorphic to β × α
.
Equations
- homeomorph.prod_comm α β = {to_equiv := equiv.prod_comm α β, continuous_to_fun := _, continuous_inv_fun := _}
(α × β) × γ
is homeomorphic to α × (β × γ)
.
Equations
- homeomorph.prod_assoc α β γ = {to_equiv := equiv.prod_assoc α β γ, continuous_to_fun := _, continuous_inv_fun := _}
α × {*}
is homeomorphic to α
.
Equations
- homeomorph.prod_punit α = {to_equiv := equiv.prod_punit α, continuous_to_fun := _, continuous_inv_fun := _}
{*} × α
is homeomorphic to α
.
Equations
If both α
and β
have a unique element, then α ≃ₜ β
.
Equations
- homeomorph.homeomorph_of_unique α β = {to_equiv := {to_fun := (equiv.equiv_of_unique α β).to_fun, inv_fun := (equiv.equiv_of_unique α β).inv_fun, left_inv := _, right_inv := _}, continuous_to_fun := _, continuous_inv_fun := _}
If each β₁ i
is homeomorphic to β₂ i
, then Π i, β₁ i
is homeomorphic to Π i, β₂ i
.
Equations
- homeomorph.Pi_congr_right F = {to_equiv := equiv.Pi_congr_right (λ (i : ι), (F i).to_equiv), continuous_to_fun := _, continuous_inv_fun := _}
ulift α
is homeomorphic to α
.
Equations
- homeomorph.ulift = {to_equiv := equiv.ulift α, continuous_to_fun := _, continuous_inv_fun := _}
(α ⊕ β) × γ
is homeomorphic to α × γ ⊕ β × γ
.
Equations
- homeomorph.sum_prod_distrib = (homeomorph.homeomorph_of_continuous_open (equiv.sum_prod_distrib α β γ).symm homeomorph.sum_prod_distrib._proof_1 homeomorph.sum_prod_distrib._proof_2).symm
α × (β ⊕ γ)
is homeomorphic to α × β ⊕ α × γ
.
Equations
- homeomorph.prod_sum_distrib = (homeomorph.prod_comm α (β ⊕ γ)).trans (homeomorph.sum_prod_distrib.trans ((homeomorph.prod_comm β α).sum_congr (homeomorph.prod_comm γ α)))
(Σ i, σ i) × β
is homeomorphic to Σ i, (σ i × β)
.
Equations
- homeomorph.sigma_prod_distrib = (homeomorph.homeomorph_of_continuous_open (equiv.sigma_prod_distrib σ β).symm homeomorph.sigma_prod_distrib._proof_1 homeomorph.sigma_prod_distrib._proof_2).symm
If ι
has a unique element, then ι → α
is homeomorphic to α
.
Equations
- homeomorph.fun_unique ι α = {to_equiv := equiv.fun_unique ι α _inst_5, continuous_to_fun := _, continuous_inv_fun := _}
Homeomorphism between dependent functions Π i : fin 2, α i
and α 0 × α 1
.
Equations
- homeomorph.pi_fin_two α = {to_equiv := pi_fin_two_equiv α, continuous_to_fun := _, continuous_inv_fun := _}
Homeomorphism between α² = fin 2 → α
and α × α
.
Equations
- homeomorph.fin_two_arrow = {to_equiv := fin_two_arrow_equiv α, continuous_to_fun := _, continuous_inv_fun := _}
A subset of a topological space is homeomorphic to its image under a homeomorphism.
Equations
- e.image s = {to_equiv := e.to_equiv.image s, continuous_to_fun := _, continuous_inv_fun := _}
set.univ α
is homeomorphic to α
.
Equations
- homeomorph.set.univ α = {to_equiv := equiv.set.univ α, continuous_to_fun := _, continuous_inv_fun := _}
s ×ˢ t
is homeomorphic to s × t
.
Equations
- homeomorph.set.prod s t = {to_equiv := equiv.set.prod s t, continuous_to_fun := _, continuous_inv_fun := _}
The topological space Π i, β i
can be split as a product by separating the indices in ι
depending on whether they satisfy a predicate p or not.
Equations
- homeomorph.pi_equiv_pi_subtype_prod p β = {to_equiv := equiv.pi_equiv_pi_subtype_prod p β (λ (a : ι), _inst_6 a), continuous_to_fun := _, continuous_inv_fun := _}
A product of topological spaces can be split as the binary product of one of the spaces and the product of all the remaining spaces.
Equations
- homeomorph.pi_split_at i β = {to_equiv := equiv.pi_split_at i β, continuous_to_fun := _, continuous_inv_fun := _}
A product of copies of a topological space can be split as the binary product of one copy and the product of all the remaining copies.
Equations
- homeomorph.fun_split_at β i = homeomorph.pi_split_at i (λ (ᾰ : ι), β)
An inducing equiv between topological spaces is a homeomorphism.
Equations
- f.to_homeomorph_of_inducing hf = {to_equiv := {to_fun := f.to_fun, inv_fun := f.inv_fun, left_inv := _, right_inv := _}, continuous_to_fun := _, continuous_inv_fun := _}
Continuous equivalences from a compact space to a T2 space are homeomorphisms.
This is not true when T2 is weakened to T1
(see continuous.homeo_of_equiv_compact_to_t2.t1_counterexample
).
Equations
- hf.homeo_of_equiv_compact_to_t2 = {to_equiv := {to_fun := f.to_fun, inv_fun := f.inv_fun, left_inv := _, right_inv := _}, continuous_to_fun := hf, continuous_inv_fun := _}