Uniform isomorphisms #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines uniform isomorphisms between two uniform spaces. They are bijections with both
directions uniformly continuous. We denote uniform isomorphisms with the notation ≃ᵤ
.
Main definitions #
uniform_equiv α β
: The type of uniform isomorphisms fromα
toβ
. This type can be denoted using the following notation:α ≃ᵤ β
.
- to_equiv : α ≃ β
- uniform_continuous_to_fun : uniform_continuous self.to_equiv.to_fun
- uniform_continuous_inv_fun : uniform_continuous self.to_equiv.inv_fun
Uniform isomorphism between α
and β
Instances for uniform_equiv
- uniform_equiv.has_sizeof_inst
- uniform_equiv.has_coe_to_fun
Inverse of a uniform isomorphism.
Equations
- h.symm = {to_equiv := h.to_equiv.symm, uniform_continuous_to_fun := _, uniform_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 uniform isomorphism.
Equations
- uniform_equiv.refl α = {to_equiv := equiv.refl α, uniform_continuous_to_fun := _, uniform_continuous_inv_fun := _}
Composition of two uniform isomorphisms.
Equations
- h₁.trans h₂ = {to_equiv := h₁.to_equiv.trans h₂.to_equiv, uniform_continuous_to_fun := _, uniform_continuous_inv_fun := _}
A uniform isomorphism as a homeomorphism.
Equations
- e.to_homeomorph = {to_equiv := {to_fun := e.to_equiv.to_fun, inv_fun := e.to_equiv.inv_fun, left_inv := _, right_inv := _}, continuous_to_fun := _, continuous_inv_fun := _}
Change the uniform equiv 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 := _}, uniform_continuous_to_fun := _, uniform_continuous_inv_fun := _}
Uniform equiv given a uniform embedding.
Equations
- uniform_equiv.of_uniform_embedding f hf = {to_equiv := equiv.of_injective f _, uniform_continuous_to_fun := _, uniform_continuous_inv_fun := _}
If two sets are equal, then they are uniformly equivalent.
Equations
- uniform_equiv.set_congr h = {to_equiv := equiv.set_congr h, uniform_continuous_to_fun := _, uniform_continuous_inv_fun := _}
Product of two uniform isomorphisms.
Equations
- h₁.prod_congr h₂ = {to_equiv := h₁.to_equiv.prod_congr h₂.to_equiv, uniform_continuous_to_fun := _, uniform_continuous_inv_fun := _}
α × β
is uniformly isomorphic to β × α
.
Equations
- uniform_equiv.prod_comm α β = {to_equiv := equiv.prod_comm α β, uniform_continuous_to_fun := _, uniform_continuous_inv_fun := _}
(α × β) × γ
is uniformly isomorphic to α × (β × γ)
.
Equations
- uniform_equiv.prod_assoc α β γ = {to_equiv := equiv.prod_assoc α β γ, uniform_continuous_to_fun := _, uniform_continuous_inv_fun := _}
α × {*}
is uniformly isomorphic to α
.
Equations
{*} × α
is uniformly isomorphic to α
.
Equations
Uniform equivalence between ulift α
and α
.
Equations
- uniform_equiv.ulift α = {to_equiv := {to_fun := equiv.ulift.to_fun, inv_fun := equiv.ulift.inv_fun, left_inv := _, right_inv := _}, uniform_continuous_to_fun := _, uniform_continuous_inv_fun := _}
If ι
has a unique element, then ι → α
is homeomorphic to α
.
Equations
- uniform_equiv.fun_unique ι α = {to_equiv := equiv.fun_unique ι α _inst_5, uniform_continuous_to_fun := _, uniform_continuous_inv_fun := _}
Uniform isomorphism between dependent functions Π i : fin 2, α i
and α 0 × α 1
.
Equations
Uniform isomorphism between α² = fin 2 → α
and α × α
.
Equations
A subset of a uniform space is uniformly isomorphic to its image under a uniform isomorphism.
Equations
- e.image s = {to_equiv := e.to_equiv.image s, uniform_continuous_to_fun := _, uniform_continuous_inv_fun := _}
A uniform inducing equiv between uniform spaces is a uniform isomorphism.
Equations
- f.to_uniform_equiv_of_uniform_inducing hf = {to_equiv := {to_fun := f.to_fun, inv_fun := f.inv_fun, left_inv := _, right_inv := _}, uniform_continuous_to_fun := _, uniform_continuous_inv_fun := _}