Isometries
We define isometries, i.e., maps between emetric spaces that preserve the edistance (on metric spaces, these are exactly the maps that preserve distances), and prove their basic properties. We also introduce isometric bijections.
An isometry (also known as isometric embedding) is a map preserving the edistance between emetric spaces, or equivalently the distance between metric space.
Equations
- isometry f = ∀ (x1 x2 : α), has_edist.edist (f x1) (f x2) = has_edist.edist x1 x2
On metric spaces, a map is an isometry if and only if it preserves distances.
An isometry preserves edistances.
An isometry preserves distances.
An isometry is injective
Any map on a subsingleton is an isometry
The composition of isometries is an isometry
An isometry is an embedding
An isometry is continuous.
The right inverse of an isometry is an isometry.
Isometries preserve the diameter in emetric spaces.
The injection from a subtype is an isometry
An isometry preserves the diameter in metric spaces.
α
and β
are isometric if there is an isometric bijection between them.
Alternative constructor for isometric bijections, taking as input an isometry, and a right inverse.
Equations
- isometric.mk' f g hfg hf = {to_equiv := {to_fun := f, inv_fun := g, left_inv := _, right_inv := hfg}, isometry_to_fun := hf}
The identity isometry of a space.
Equations
- isometric.refl α = {to_equiv := {to_fun := (equiv.refl α).to_fun, inv_fun := (equiv.refl α).inv_fun, left_inv := _, right_inv := _}, isometry_to_fun := _}
The composition of two isometric isomorphisms, as an isometric isomorphism.
The inverse of an isometric isomorphism, as an isometric isomorphism.
The (bundled) homeomorphism associated to an isometric isomorphism.
Equations
- h.to_homeomorph = {to_equiv := h.to_equiv, continuous_to_fun := _, continuous_inv_fun := _}
The group of isometries.
Equations
- isometric.group = {mul := λ (e₁ e₂ : α ≃ᵢ α), e₁.trans e₂, mul_assoc := _, one := isometric.refl α _inst_1, one_mul := _, mul_one := _, inv := isometric.symm _inst_1, mul_left_inv := _}
Addition y ↦ y + x
as an isometry
.
Equations
- isometric.add_right x = {to_equiv := {to_fun := (equiv.add_right x).to_fun, inv_fun := (equiv.add_right x).inv_fun, left_inv := _, right_inv := _}, isometry_to_fun := _}
Addition y ↦ x + y
as an isometry
.
Equations
- isometric.add_left x = {to_equiv := equiv.add_left x, isometry_to_fun := _}
Negation x ↦ -x
as an isometry
.
Equations
- isometric.neg G = {to_equiv := equiv.neg G (add_comm_group.to_add_group G), isometry_to_fun := _}
An isometry induces an isometric isomorphism between the source space and the range of the isometry.
Equations
- h.isometric_on_range = {to_equiv := {to_fun := (equiv.set.range f _).to_fun, inv_fun := (equiv.set.range f _).inv_fun, left_inv := _, right_inv := _}, isometry_to_fun := _}
In a normed algebra, the inclusion of the base field in the extended field is an isometry.
In this section, we show that any separable metric space can be embedded isometrically in ℓ^∞(ℝ)
A metric space can be embedded in l^∞(ℝ)
via the distances to points in
a fixed countable set, if this set is dense. This map is given in the next definition,
without density assumptions.
Equations
- Kuratowski_embedding.embedding_of_subset x a = bounded_continuous_function.of_normed_group_discrete (λ (n : ℕ), has_dist.dist a (x n) - has_dist.dist (x 0) (x n)) (has_dist.dist a (x 0)) _
The embedding map is always a semi-contraction.
When the reference set is dense, the embedding map is an isometry on its image.
Every separable metric space embeds isometrically in ℓ_infty_ℝ.
The Kuratowski embedding is an isometric embedding of a separable metric space in ℓ^∞(ℝ)
Equations
The Kuratowski embedding is an isometry
Version of the Kuratowski embedding for nonempty compacts