Documentation

Mathlib.Topology.MetricSpace.Isometry

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.

Since a lot of elementary properties don't require eq_of_dist_eq_zero we start setting up the theory for PseudoMetricSpace and we specialize to MetricSpace when needed.

def Isometry {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (f : αβ) :

An isometry (also known as isometric embedding) is a map preserving the edistance between pseudoemetric spaces, or equivalently the distance between pseudometric space.

Equations
theorem isometry_iff_nndist_eq {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] {f : αβ} :
Isometry f ∀ (x y : α), nndist (f x) (f y) = nndist x y

On pseudometric spaces, a map is an isometry if and only if it preserves nonnegative distances.

theorem isometry_iff_dist_eq {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] {f : αβ} :
Isometry f ∀ (x y : α), dist (f x) (f y) = dist x y

On pseudometric spaces, a map is an isometry if and only if it preserves distances.

theorem Isometry.dist_eq {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] {f : αβ} :
Isometry f∀ (x y : α), dist (f x) (f y) = dist x y

An isometry preserves distances.

theorem Isometry.of_dist_eq {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] {f : αβ} :
(∀ (x y : α), dist (f x) (f y) = dist x y)Isometry f

A map that preserves distances is an isometry

theorem Isometry.nndist_eq {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] {f : αβ} :
Isometry f∀ (x y : α), nndist (f x) (f y) = nndist x y

An isometry preserves non-negative distances.

theorem Isometry.of_nndist_eq {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] {f : αβ} :
(∀ (x y : α), nndist (f x) (f y) = nndist x y)Isometry f

A map that preserves non-negative distances is an isometry.

theorem Isometry.edist_eq {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (hf : Isometry f) (x y : α) :
edist (f x) (f y) = edist x y

An isometry preserves edistances.

theorem Isometry.lipschitz {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (h : Isometry f) :
theorem Isometry.antilipschitz {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (h : Isometry f) :
theorem isometry_subsingleton {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {f : αβ} [Subsingleton α] :

Any map on a subsingleton is an isometry

The identity is an isometry

theorem Isometry.prod_map {α : Type u} {β : Type v} {γ : Type w} [PseudoEMetricSpace α] [PseudoEMetricSpace β] [PseudoEMetricSpace γ] {δ : Type u_2} [PseudoEMetricSpace δ] {f : αβ} {g : γδ} (hf : Isometry f) (hg : Isometry g) :
theorem Isometry.piMap {ι : Type u_4} [Fintype ι] {α : ιType u_2} {β : ιType u_3} [(i : ι) → PseudoEMetricSpace (α i)] [(i : ι) → PseudoEMetricSpace (β i)] (f : (i : ι) → α iβ i) (hf : ∀ (i : ι), Isometry (f i)) :
@[deprecated Isometry.piMap (since := "2024-10-06")]
theorem isometry_dcomp {ι : Type u_4} [Fintype ι] {α : ιType u_2} {β : ιType u_3} [(i : ι) → PseudoEMetricSpace (α i)] [(i : ι) → PseudoEMetricSpace (β i)] (f : (i : ι) → α iβ i) (hf : ∀ (i : ι), Isometry (f i)) :

Alias of Isometry.piMap.

theorem Isometry.comp {α : Type u} {β : Type v} {γ : Type w} [PseudoEMetricSpace α] [PseudoEMetricSpace β] [PseudoEMetricSpace γ] {g : βγ} {f : αβ} (hg : Isometry g) (hf : Isometry f) :

The composition of isometries is an isometry.

theorem Isometry.uniformContinuous {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (hf : Isometry f) :

An isometry from a metric space is a uniform continuous map

theorem Isometry.isUniformInducing {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (hf : Isometry f) :

An isometry from a metric space is a uniform inducing map

@[deprecated Isometry.isUniformInducing (since := "2024-10-05")]
theorem Isometry.uniformInducing {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (hf : Isometry f) :

Alias of Isometry.isUniformInducing.


An isometry from a metric space is a uniform inducing map

theorem Isometry.tendsto_nhds_iff {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {ι : Type u_2} {f : αβ} {g : ια} {a : Filter ι} {b : α} (hf : Isometry f) :
Filter.Tendsto g a (nhds b) Filter.Tendsto (f g) a (nhds (f b))
theorem Isometry.continuous {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (hf : Isometry f) :

An isometry is continuous.

theorem Isometry.right_inv {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {f : αβ} {g : βα} (h : Isometry f) (hg : Function.RightInverse g f) :

The right inverse of an isometry is an isometry.

theorem Isometry.preimage_emetric_closedBall {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (h : Isometry f) (x : α) (r : ENNReal) :
theorem Isometry.preimage_emetric_ball {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (h : Isometry f) (x : α) (r : ENNReal) :
theorem Isometry.ediam_image {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (hf : Isometry f) (s : Set α) :

Isometries preserve the diameter in pseudoemetric spaces.

theorem Isometry.mapsTo_emetric_ball {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (hf : Isometry f) (x : α) (r : ENNReal) :
theorem Isometry.mapsTo_emetric_closedBall {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (hf : Isometry f) (x : α) (r : ENNReal) :

The injection from a subtype is an isometry

theorem Isometry.comp_continuousOn_iff {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {f : αβ} {γ : Type u_2} [TopologicalSpace γ] (hf : Isometry f) {g : γα} {s : Set γ} :
theorem Isometry.comp_continuous_iff {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {f : αβ} {γ : Type u_2} [TopologicalSpace γ] (hf : Isometry f) {g : γα} :
theorem Isometry.injective {α : Type u} {β : Type v} [EMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (h : Isometry f) :

An isometry from an emetric space is injective

theorem Isometry.isUniformEmbedding {α : Type u} {β : Type v} [EMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (hf : Isometry f) :

An isometry from an emetric space is a uniform embedding

@[deprecated Isometry.isUniformEmbedding (since := "2024-10-01")]
theorem Isometry.uniformEmbedding {α : Type u} {β : Type v} [EMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (hf : Isometry f) :

Alias of Isometry.isUniformEmbedding.


An isometry from an emetric space is a uniform embedding

theorem Isometry.isEmbedding {α : Type u} {β : Type v} [EMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (hf : Isometry f) :

An isometry from an emetric space is an embedding

@[deprecated Isometry.isEmbedding (since := "2024-10-26")]
theorem Isometry.embedding {α : Type u} {β : Type v} [EMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (hf : Isometry f) :

Alias of Isometry.isEmbedding.


An isometry from an emetric space is an embedding

theorem Isometry.isClosedEmbedding {α : Type u} {γ : Type w} [EMetricSpace α] [CompleteSpace α] [EMetricSpace γ] {f : αγ} (hf : Isometry f) :

An isometry from a complete emetric space is a closed embedding

@[deprecated Isometry.isClosedEmbedding (since := "2024-10-20")]
theorem Isometry.closedEmbedding {α : Type u} {γ : Type w} [EMetricSpace α] [CompleteSpace α] [EMetricSpace γ] {f : αγ} (hf : Isometry f) :

Alias of Isometry.isClosedEmbedding.


An isometry from a complete emetric space is a closed embedding

theorem Isometry.diam_image {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] {f : αβ} (hf : Isometry f) (s : Set α) :

An isometry preserves the diameter in pseudometric spaces.

theorem Isometry.preimage_setOf_dist {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] {f : αβ} (hf : Isometry f) (x : α) (p : Prop) :
f ⁻¹' {y : β | p (dist y (f x))} = {y : α | p (dist y x)}
theorem Isometry.preimage_closedBall {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] {f : αβ} (hf : Isometry f) (x : α) (r : ) :
theorem Isometry.preimage_ball {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] {f : αβ} (hf : Isometry f) (x : α) (r : ) :
theorem Isometry.preimage_sphere {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] {f : αβ} (hf : Isometry f) (x : α) (r : ) :
theorem Isometry.mapsTo_ball {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] {f : αβ} (hf : Isometry f) (x : α) (r : ) :
theorem Isometry.mapsTo_sphere {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] {f : αβ} (hf : Isometry f) (x : α) (r : ) :
theorem Isometry.mapsTo_closedBall {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] {f : αβ} (hf : Isometry f) (x : α) (r : ) :
theorem IsUniformEmbedding.to_isometry {α : Type u_2} {β : Type u_3} [UniformSpace α] [MetricSpace β] {f : αβ} (h : IsUniformEmbedding f) :

A uniform embedding from a uniform space to a metric space is an isometry with respect to the induced metric space structure on the source space.

@[deprecated IsUniformEmbedding.to_isometry (since := "2024-10-01")]
theorem UniformEmbedding.to_isometry {α : Type u_2} {β : Type u_3} [UniformSpace α] [MetricSpace β] {f : αβ} (h : IsUniformEmbedding f) :

Alias of IsUniformEmbedding.to_isometry.


A uniform embedding from a uniform space to a metric space is an isometry with respect to the induced metric space structure on the source space.

theorem Topology.IsEmbedding.to_isometry {α : Type u_2} {β : Type u_3} [TopologicalSpace α] [MetricSpace β] {f : αβ} (h : IsEmbedding f) :

An embedding from a topological space to a metric space is an isometry with respect to the induced metric space structure on the source space.

@[deprecated Topology.IsEmbedding.to_isometry (since := "2024-10-26")]
theorem Embedding.to_isometry {α : Type u_2} {β : Type u_3} [TopologicalSpace α] [MetricSpace β] {f : αβ} (h : Topology.IsEmbedding f) :

Alias of Topology.IsEmbedding.to_isometry.


An embedding from a topological space to a metric space is an isometry with respect to the induced metric space structure on the source space.

theorem PseudoEMetricSpace.isometry_induced {α : Type u} {β : Type v} (f : αβ) [m : PseudoEMetricSpace β] :
theorem PsuedoMetricSpace.isometry_induced {α : Type u} {β : Type v} (f : αβ) [m : PseudoMetricSpace β] :
theorem EMetricSpace.isometry_induced {α : Type u} {β : Type v} (f : αβ) (hf : Function.Injective f) [m : EMetricSpace β] :
theorem MetricSpace.isometry_induced {α : Type u} {β : Type v} (f : αβ) (hf : Function.Injective f) [m : MetricSpace β] :
structure IsometryEquiv (α : Type u) (β : Type v) [PseudoEMetricSpace α] [PseudoEMetricSpace β] extends α β :
Type (max u v)

α and β are isometric if there is an isometric bijection between them.

Instances For

α and β are isometric if there is an isometric bijection between them.

Equations
@[simp]
theorem IsometryEquiv.toEquiv_inj {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {e₁ e₂ : α ≃ᵢ β} :
e₁.toEquiv = e₂.toEquiv e₁ = e₂
instance IsometryEquiv.instEquivLike {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] :
EquivLike (α ≃ᵢ β) α β
Equations
theorem IsometryEquiv.coe_eq_toEquiv {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) (a : α) :
h a = h.toEquiv a
@[simp]
theorem IsometryEquiv.coe_toEquiv {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) :
h.toEquiv = h
@[simp]
theorem IsometryEquiv.coe_mk {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (e : α β) (h : Isometry e.toFun) :
{ toEquiv := e, isometry_toFun := h } = e
theorem IsometryEquiv.isometry {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) :
theorem IsometryEquiv.edist_eq {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) (x y : α) :
edist (h x) (h y) = edist x y
theorem IsometryEquiv.dist_eq {α : Type u_2} {β : Type u_3} [PseudoMetricSpace α] [PseudoMetricSpace β] (h : α ≃ᵢ β) (x y : α) :
dist (h x) (h y) = dist x y
theorem IsometryEquiv.nndist_eq {α : Type u_2} {β : Type u_3} [PseudoMetricSpace α] [PseudoMetricSpace β] (h : α ≃ᵢ β) (x y : α) :
nndist (h x) (h y) = nndist x y
theorem IsometryEquiv.continuous {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) :
@[simp]
theorem IsometryEquiv.ediam_image {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) (s : Set α) :
theorem IsometryEquiv.ext {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] h₁ h₂ : α ≃ᵢ β (H : ∀ (x : α), h₁ x = h₂ x) :
h₁ = h₂
def IsometryEquiv.mk' {β : Type v} [PseudoEMetricSpace β] {α : Type u} [EMetricSpace α] (f : αβ) (g : βα) (hfg : ∀ (x : β), f (g x) = x) (hf : Isometry f) :
α ≃ᵢ β

Alternative constructor for isometric bijections, taking as input an isometry, and a right inverse.

Equations
  • IsometryEquiv.mk' f g hfg hf = { toFun := f, invFun := g, left_inv := , right_inv := hfg, isometry_toFun := hf }

The identity isometry of a space.

Equations
def IsometryEquiv.trans {α : Type u} {β : Type v} {γ : Type w} [PseudoEMetricSpace α] [PseudoEMetricSpace β] [PseudoEMetricSpace γ] (h₁ : α ≃ᵢ β) (h₂ : β ≃ᵢ γ) :
α ≃ᵢ γ

The composition of two isometric isomorphisms, as an isometric isomorphism.

Equations
@[simp]
theorem IsometryEquiv.trans_apply {α : Type u} {β : Type v} {γ : Type w} [PseudoEMetricSpace α] [PseudoEMetricSpace β] [PseudoEMetricSpace γ] (h₁ : α ≃ᵢ β) (h₂ : β ≃ᵢ γ) (x : α) :
(h₁.trans h₂) x = h₂ (h₁ x)
def IsometryEquiv.symm {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) :
β ≃ᵢ α

The inverse of an isometric isomorphism, as an isometric isomorphism.

Equations
  • h.symm = { toEquiv := h.symm, isometry_toFun := }
def IsometryEquiv.Simps.apply {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) :
αβ

See Note [custom simps projection]. We need to specify this projection explicitly in this case, because it is a composition of multiple projections.

Equations
def IsometryEquiv.Simps.symm_apply {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) :
βα

See Note [custom simps projection]

Equations
@[simp]
theorem IsometryEquiv.symm_symm {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) :
h.symm.symm = h
@[simp]
theorem IsometryEquiv.apply_symm_apply {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) (y : β) :
h (h.symm y) = y
@[simp]
theorem IsometryEquiv.symm_apply_apply {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) (x : α) :
h.symm (h x) = x
theorem IsometryEquiv.symm_apply_eq {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) {x : α} {y : β} :
h.symm y = x y = h x
theorem IsometryEquiv.eq_symm_apply {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) {x : α} {y : β} :
x = h.symm y h x = y
theorem IsometryEquiv.symm_comp_self {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) :
h.symm h = id
theorem IsometryEquiv.self_comp_symm {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) :
h h.symm = id
@[simp]
theorem IsometryEquiv.symm_trans_apply {α : Type u} {β : Type v} {γ : Type w} [PseudoEMetricSpace α] [PseudoEMetricSpace β] [PseudoEMetricSpace γ] (h₁ : α ≃ᵢ β) (h₂ : β ≃ᵢ γ) (x : γ) :
(h₁.trans h₂).symm x = h₁.symm (h₂.symm x)
@[simp]
theorem IsometryEquiv.ediam_preimage {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) (s : Set β) :
@[simp]
theorem IsometryEquiv.preimage_emetric_ball {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) (x : β) (r : ENNReal) :
@[simp]
theorem IsometryEquiv.image_emetric_ball {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) (x : α) (r : ENNReal) :
h '' EMetric.ball x r = EMetric.ball (h x) r
@[simp]
theorem IsometryEquiv.image_emetric_closedBall {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) (x : α) (r : ENNReal) :
def IsometryEquiv.toHomeomorph {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) :
α ≃ₜ β

The (bundled) homeomorphism associated to an isometric isomorphism.

Equations
@[simp]
theorem IsometryEquiv.coe_toHomeomorph {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] (h : α ≃ᵢ β) :
h.toHomeomorph = h
@[simp]
@[simp]
theorem IsometryEquiv.comp_continuousOn_iff {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {γ : Type u_2} [TopologicalSpace γ] (h : α ≃ᵢ β) {f : γα} {s : Set γ} :
@[simp]
theorem IsometryEquiv.comp_continuous_iff {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {γ : Type u_2} [TopologicalSpace γ] (h : α ≃ᵢ β) {f : γα} :
@[simp]
theorem IsometryEquiv.comp_continuous_iff' {α : Type u} {β : Type v} [PseudoEMetricSpace α] [PseudoEMetricSpace β] {γ : Type u_2} [TopologicalSpace γ] (h : α ≃ᵢ β) {f : βγ} :

The group of isometries.

Equations
@[simp]
theorem IsometryEquiv.coe_one {α : Type u} [PseudoEMetricSpace α] :
1 = id
@[simp]
theorem IsometryEquiv.coe_mul {α : Type u} [PseudoEMetricSpace α] (e₁ e₂ : α ≃ᵢ α) :
⇑(e₁ * e₂) = e₁ e₂
theorem IsometryEquiv.mul_apply {α : Type u} [PseudoEMetricSpace α] (e₁ e₂ : α ≃ᵢ α) (x : α) :
(e₁ * e₂) x = e₁ (e₂ x)
@[simp]
theorem IsometryEquiv.inv_apply_self {α : Type u} [PseudoEMetricSpace α] (e : α ≃ᵢ α) (x : α) :
e⁻¹ (e x) = x
@[simp]
theorem IsometryEquiv.apply_inv_self {α : Type u} [PseudoEMetricSpace α] (e : α ≃ᵢ α) (x : α) :
e (e⁻¹ x) = x
def IsometryEquiv.piCongrLeft' {ι : Type u_1} {ι' : Type u_2} [Fintype ι] [Fintype ι'] {Y : ιType u_3} [(j : ι) → PseudoEMetricSpace (Y j)] (e : ι ι') :
((i : ι) → Y i) ≃ᵢ ((j : ι') → Y (e.symm j))

The natural isometry ∀ i, Y i ≃ᵢ ∀ j, Y (e.symm j) obtained from a bijection ι ≃ ι' of fintypes. Equiv.piCongrLeft' as an IsometryEquiv.

Equations
@[simp]
theorem IsometryEquiv.piCongrLeft'_symm_apply {ι : Type u_1} {ι' : Type u_2} [Fintype ι] [Fintype ι'] {Y : ιType u_3} [(j : ι) → PseudoEMetricSpace (Y j)] (e : ι ι') (f : (b : ι') → Y (e.symm b)) (x : ι) :
(piCongrLeft' e).symm f x = f (e x)
@[simp]
theorem IsometryEquiv.piCongrLeft'_apply {ι : Type u_1} {ι' : Type u_2} [Fintype ι] [Fintype ι'] {Y : ιType u_3} [(j : ι) → PseudoEMetricSpace (Y j)] (e : ι ι') (f : (a : ι) → Y a) (x : ι') :
(piCongrLeft' e) f x = f (e.symm x)
def IsometryEquiv.piCongrLeft {ι : Type u_1} {ι' : Type u_2} [Fintype ι] [Fintype ι'] {Y : ι'Type u_3} [(j : ι') → PseudoEMetricSpace (Y j)] (e : ι ι') :
((i : ι) → Y (e i)) ≃ᵢ ((j : ι') → Y j)

The natural isometry ∀ i, Y (e i) ≃ᵢ ∀ j, Y j obtained from a bijection ι ≃ ι' of fintypes. Equiv.piCongrLeft as an IsometryEquiv.

Equations
@[simp]
theorem IsometryEquiv.piCongrLeft_apply {ι : Type u_1} {ι' : Type u_2} [Fintype ι] [Fintype ι'] {Y : ι'Type u_3} [(j : ι') → PseudoEMetricSpace (Y j)] (e : ι ι') (a✝ : (j : ι) → Y (e.symm.symm j)) (i : ι') :
(piCongrLeft e) a✝ i = (piCongrLeft' e.symm).symm a✝ i
@[simp]
theorem IsometryEquiv.piCongrLeft_symm_apply {ι : Type u_1} {ι' : Type u_2} [Fintype ι] [Fintype ι'] {Y : ι'Type u_3} [(j : ι') → PseudoEMetricSpace (Y j)] (e : ι ι') (a✝ : (i : ι') → Y i) (j : ι) :
(piCongrLeft e).symm a✝ j = (piCongrLeft' e.symm) a✝ j
def IsometryEquiv.sumArrowIsometryEquivProdArrow {α : Type u} {β : Type v} {γ : Type w} [PseudoEMetricSpace γ] [Fintype α] [Fintype β] :
(α βγ) ≃ᵢ (αγ) × (βγ)

The natural isometry (α ⊕ β → γ) ≃ᵢ (α → γ) × (β → γ) between the type of maps on a sum of fintypes α ⊕ β and the pairs of functions on the types α and β. Equiv.sumArrowEquivProdArrow as an IsometryEquiv.

Equations
@[simp]
theorem IsometryEquiv.sumArrowIsometryEquivProdArrow_symm_apply {α : Type u} {β : Type v} {γ : Type w} [PseudoEMetricSpace γ] [Fintype α] [Fintype β] (p : (αγ) × (βγ)) (a✝ : α β) :
theorem Fin.edist_append_eq_max_edist {α : Type u} [PseudoEMetricSpace α] (m n : ) {x x2 : Fin mα} {y y2 : Fin nα} :
edist (append x y) (append x2 y2) = edist x x2 edist y y2
def Fin.appendIsometry {α : Type u} [PseudoEMetricSpace α] (m n : ) :
(Fin mα) × (Fin nα) ≃ᵢ (Fin (m + n)α)

The natural IsometryEquiv between (Fin m → α) × (Fin n → α) and Fin (m + n) → α. Fin.appendEquiv as an IsometryEquiv.

Equations
@[simp]
theorem Fin.appendIsometry_symm_apply {α : Type u} [PseudoEMetricSpace α] (m n : ) (f : Fin (m + n)α) :
(appendIsometry m n).symm f = (fun (i : Fin m) => f (castAdd n i), fun (i : Fin n) => f (natAdd m i))
@[simp]
theorem Fin.appendIsometry_apply {α : Type u} [PseudoEMetricSpace α] (m n : ) (fg : (Fin mα) × (Fin nα)) (a✝ : Fin (m + n)) :
(appendIsometry m n) fg a✝ = append fg.1 fg.2 a✝
def IsometryEquiv.funUnique (ι : Type u_1) (α : Type u) [PseudoEMetricSpace α] [Unique ι] [Fintype ι] :
(ια) ≃ᵢ α

Equiv.funUnique as an IsometryEquiv.

Equations
@[simp]
theorem IsometryEquiv.funUnique_apply (ι : Type u_1) (α : Type u) [PseudoEMetricSpace α] [Unique ι] [Fintype ι] (f : (i : ι) → (fun (a : ι) => α) i) :
(funUnique ι α) f = f default
@[simp]
theorem IsometryEquiv.funUnique_symm_apply (ι : Type u_1) (α : Type u) [PseudoEMetricSpace α] [Unique ι] [Fintype ι] (x : α) (i : ι) :
(funUnique ι α).symm x i = x
def IsometryEquiv.piFinTwo (α : Fin 2Type u_2) [(i : Fin 2) → PseudoEMetricSpace (α i)] :
((i : Fin 2) → α i) ≃ᵢ α 0 × α 1

piFinTwoEquiv as an IsometryEquiv.

Equations
@[simp]
theorem IsometryEquiv.piFinTwo_apply (α : Fin 2Type u_2) [(i : Fin 2) → PseudoEMetricSpace (α i)] (f : (i : Fin 2) → α i) :
(piFinTwo α) f = (f 0, f 1)
@[simp]
theorem IsometryEquiv.piFinTwo_symm_apply (α : Fin 2Type u_2) [(i : Fin 2) → PseudoEMetricSpace (α i)] (p : α 0 × α 1) (i : Fin (1 + 1)) :
@[simp]
theorem IsometryEquiv.diam_image {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] (h : α ≃ᵢ β) (s : Set α) :
@[simp]
theorem IsometryEquiv.diam_preimage {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] (h : α ≃ᵢ β) (s : Set β) :
@[simp]
theorem IsometryEquiv.preimage_ball {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] (h : α ≃ᵢ β) (x : β) (r : ) :
@[simp]
theorem IsometryEquiv.preimage_sphere {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] (h : α ≃ᵢ β) (x : β) (r : ) :
@[simp]
theorem IsometryEquiv.preimage_closedBall {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] (h : α ≃ᵢ β) (x : β) (r : ) :
@[simp]
theorem IsometryEquiv.image_ball {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] (h : α ≃ᵢ β) (x : α) (r : ) :
h '' Metric.ball x r = Metric.ball (h x) r
@[simp]
theorem IsometryEquiv.image_sphere {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] (h : α ≃ᵢ β) (x : α) (r : ) :
h '' Metric.sphere x r = Metric.sphere (h x) r
@[simp]
theorem IsometryEquiv.image_closedBall {α : Type u} {β : Type v} [PseudoMetricSpace α] [PseudoMetricSpace β] (h : α ≃ᵢ β) (x : α) (r : ) :
def Isometry.isometryEquivOnRange {α : Type u} {β : Type v} [EMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (h : Isometry f) :
α ≃ᵢ (Set.range f)

An isometry induces an isometric isomorphism between the source space and the range of the isometry.

Equations
@[simp]
theorem Isometry.isometryEquivOnRange_apply {α : Type u} {β : Type v} [EMetricSpace α] [PseudoEMetricSpace β] {f : αβ} (h : Isometry f) (a : α) :
h.isometryEquivOnRange a = f a,
theorem Isometry.lipschitzWith_iff {α : Type u_2} {β : Type u_3} {γ : Type u_4} [PseudoEMetricSpace α] [PseudoEMetricSpace β] [PseudoEMetricSpace γ] {f : αβ} {g : βγ} (K : NNReal) (h : Isometry g) :

Post-composition by an isometry does not change the Lipschitz-property of a function.