Documentation

Mathlib.Topology.MetricSpace.Completion

The completion of a metric space #

Completion of uniform spaces are already defined in Topology.UniformSpace.Completion. We show here that the uniform space completion of a metric space inherits a metric space structure, by extending the distance to the completion and checking that it is indeed a distance, and that it defines the same uniformity as the already defined uniform structure on the completion

The distance on the completion is obtained by extending the distance on the original space, by uniform continuity.

Equations

The new distance is uniformly continuous.

theorem UniformSpace.Completion.continuous_dist {α : Type u} {β : Type v} [PseudoMetricSpace α] [TopologicalSpace β] {f : βUniformSpace.Completion α} {g : βUniformSpace.Completion α} (hf : Continuous f) (hg : Continuous g) :
Continuous fun (x : β) => dist (f x) (g x)

The new distance is continuous.

@[simp]
theorem UniformSpace.Completion.dist_eq {α : Type u} [PseudoMetricSpace α] (x : α) (y : α) :
dist (α x) (α y) = dist x y

The new distance is an extension of the original distance.

Elements of the uniformity (defined generally for completions) can be characterized in terms of the distance.

Reformulate Completion.mem_uniformity_dist in terms that are suitable for the definition of the metric space structure.

Metric space structure on the completion of a pseudo_metric space.

Equations
@[deprecated eq_of_dist_eq_zero]

The embedding of a metric space in its completion is an isometry.

@[simp]
theorem UniformSpace.Completion.edist_eq {α : Type u} [PseudoMetricSpace α] (x : α) (y : α) :
edist (α x) (α y) = edist x y