Extended metric spaces
This file is devoted to the definition and study of emetric_spaces
, i.e., metric
spaces in which the distance is allowed to take the value ∞. This extended distance is
called edist
, and takes values in ennreal
.
Many definitions and theorems expected on emetric spaces are already introduced on uniform spaces and topological spaces. For example: open and closed sets, compactness, completeness, continuity and uniform continuity
The class emetric_space
therefore extends uniform_space
(and topological_space
).
Characterizing uniformities associated to a (generalized) distance function D
in terms of the elements of the uniformity.
- edist : α → α → ennreal
Creating a uniform space from an extended distance.
Equations
- uniform_space_of_edist edist edist_self edist_comm edist_triangle = uniform_space.of_core {uniformity := ⨅ (ε : ennreal) (H : ε > 0), filter.principal {p : α × α | edist p.fst p.snd < ε}, refl := _, symm := _, comp := _}
- to_has_edist : has_edist α
- edist_self : ∀ (x : α), has_edist.edist x x = 0
- eq_of_edist_eq_zero : ∀ {x y : α}, has_edist.edist x y = 0 → x = y
- edist_comm : ∀ (x y : α), has_edist.edist x y = has_edist.edist y x
- edist_triangle : ∀ (x y z : α), has_edist.edist x z ≤ has_edist.edist x y + has_edist.edist y z
- to_uniform_space : uniform_space α
- uniformity_edist : (uniformity α = ⨅ (ε : ennreal) (H : ε > 0), filter.principal {p : α × α | has_edist.edist p.fst p.snd < ε}) . "control_laws_tac"
Extended metric spaces, with an extended distance edist
possibly taking the
value ∞
Each emetric space induces a canonical uniform_space
and hence a canonical topological_space
.
This is enforced in the type class definition, by extending the uniform_space
structure. When
instantiating an emetric_space
structure, the uniformity fields are not necessary, they will be
filled in by default. There is a default value for the uniformity, that can be substituted
in cases of interest, for instance when instantiating an emetric_space
structure
on a product.
Continuity of edist
is proved in topology.instances.ennreal
Characterize the equality of points by the vanishing of their extended distance
Triangle inequality for the extended distance
The triangle (polygon) inequality for sequences of points; finset.Ico
version.
The triangle (polygon) inequality for sequences of points; finset.range
version.
A version of edist_le_Ico_sum_edist
with each intermediate distance replaced
with an upper estimate.
A version of edist_le_range_sum_edist
with each intermediate distance replaced
with an upper estimate.
Two points coincide if their distance is < ε
for all positive ε
Reformulation of the uniform structure in terms of the extended distance
Characterization of the elements of the uniformity in terms of the extended distance
Given f : β → ennreal
, if f
sends {i | p i}
to a set of positive numbers
accumulating to zero, then f i
-neighborhoods of the diagonal form a basis of 𝓤 α
.
For specific bases see uniformity_basis_edist
, uniformity_basis_edist'
,
uniformity_basis_edist_nnreal
, and uniformity_basis_edist_inv_nat
.
Given f : β → ennreal
, if f
sends {i | p i}
to a set of positive numbers
accumulating to zero, then closed f i
-neighborhoods of the diagonal form a basis of 𝓤 α
.
For specific bases see uniformity_basis_edist_le
and uniformity_basis_edist_le'
.
Fixed size neighborhoods of the diagonal belong to the uniform structure
ε-δ characterization of uniform continuity on emetric spaces
ε-δ characterization of uniform embeddings on emetric spaces
A map between emetric spaces is a uniform embedding if and only if the edistance between f x
and f y
is controlled in terms of the distance between x
and y
and conversely.
A very useful criterion to show that a space is complete is to show that all sequences
which satisfy a bound of the form edist (u n) (u m) < B N
for all n m ≥ N
are
converging. This is often applied for B N = 2^{-N}
, i.e., with a very fast convergence to
0
, which makes it possible to use arguments of converging series, while this is impossible
to do in general for arbitrary Cauchy sequences.
A sequentially complete emetric space is complete.
Expressing locally uniform convergence on a set using edist
.
Expressing uniform convergence on a set using edist
.
Expressing locally uniform convergence using edist
.
Expressing uniform convergence using edist
.
An emetric space is separated
Equations
Auxiliary function to replace the uniformity on an emetric space with a uniformity which is equal to the original one, but maybe not defeq. This is useful if one wants to construct an emetric space with a specified uniformity. See Note [forgetful inheritance] explaining why having definitionally the right uniformity is often important.
Equations
- m.replace_uniformity H = {to_has_edist := {edist := has_edist.edist emetric_space.to_has_edist}, edist_self := _, eq_of_edist_eq_zero := _, edist_comm := _, edist_triangle := _, to_uniform_space := U, uniformity_edist := _}
The extended metric induced by an injective function taking values in an emetric space.
Equations
- emetric_space.induced f hf m = {to_has_edist := {edist := λ (x y : α), has_edist.edist (f x) (f y)}, edist_self := _, eq_of_edist_eq_zero := _, edist_comm := _, edist_triangle := _, to_uniform_space := uniform_space.comap f emetric_space.to_uniform_space, uniformity_edist := _}
Emetric space instance on subsets of emetric spaces
Equations
- subtype.emetric_space = emetric_space.induced coe subtype.emetric_space._proof_1 t
The extended distance on a subset of an emetric space is the restriction of the original distance, by definition
The product of two emetric spaces, with the max distance, is an extended metric spaces. We make sure that the uniform structure thus constructed is the one corresponding to the product of uniform spaces, to avoid diamond problems.
Equations
- prod.emetric_space_max = {to_has_edist := {edist := λ (x y : α × β), max (has_edist.edist x.fst y.fst) (has_edist.edist x.snd y.snd)}, edist_self := _, eq_of_edist_eq_zero := _, edist_comm := _, edist_triangle := _, to_uniform_space := prod.uniform_space emetric_space.to_uniform_space', uniformity_edist := _}
The product of a finite number of emetric spaces, with the max distance, is still an emetric space. This construction would also work for infinite products, but it would not give rise to the product topology. Hence, we only formalize it in the good situation of finitely many spaces.
Equations
- emetric_space_pi = {to_has_edist := {edist := λ (f g : Π (b : β), π b), finset.univ.sup (λ (b : β), has_edist.edist (f b) (g b))}, edist_self := _, eq_of_edist_eq_zero := _, edist_comm := _, edist_triangle := _, to_uniform_space := Pi.uniform_space (λ (b : β), π b) (λ (i : β), emetric_space.to_uniform_space'), uniformity_edist := _}
emetric.ball x ε
is the set of all points y
with edist y x < ε
Equations
- emetric.ball x ε = {y : α | has_edist.edist y x < ε}
emetric.closed_ball x ε
is the set of all points y
with edist y x ≤ ε
Equations
- emetric.closed_ball x ε = {y : α | has_edist.edist y x ≤ ε}
Relation “two points are at a finite edistance” is an equivalence relation.
Equations
- emetric.edist_lt_top_setoid = {r := λ (x y : α), has_edist.edist x y < ⊤, iseqv := _}
ε-characterization of the closure in emetric spaces
In an emetric space, Cauchy sequences are characterized by the fact that, eventually, the edistance between its elements is arbitrarily small
A variation around the emetric characterization of Cauchy sequences
A variation of the emetric characterization of Cauchy sequences that deals with
nnreal
upper bounds.
A compact set in an emetric space is separable, i.e., it is the closure of a countable set
Equations
- _ = _
A separable emetric space is second countable: one obtains a countable basis by taking the balls centered at points in a dense subset, and with rational radii. We do not register this as an instance, as there is already an instance going in the other direction from second countable spaces to separable spaces, and we want to avoid loops.
The diameter of a set in an emetric space, named emetric.diam
Equations
- emetric.diam s = ⨆ (x : α) (H : x ∈ s) (y : α) (H : y ∈ s), has_edist.edist x y
If two points belong to some set, their edistance is bounded by the diameter of the set
If the distance between any two points in a set is bounded by some constant, this constant bounds the diameter.
The diameter of a subsingleton vanishes.
The diameter of the empty set vanishes
The diameter of a singleton vanishes
The diameter is monotonous with respect to inclusion
The diameter of a union is controlled by the diameter of the sets, and the edistance between two points in the sets.