mathlib3 documentation

topology.metric_space.gluing

Metric space gluing #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

Gluing two metric spaces along a common subset. Formally, we are given

     Φ
  Z ---> X
  |
  
  v
  Y

where hΦ : isometry Φ and hΨ : isometry Ψ. We want to complete the square by a space glue_space hΦ hΨ and two isometries to_glue_l hΦ hΨ and to_glue_r hΦ hΨ that make the square commute. We start by defining a predistance on the disjoint union X ⊕ Y, for which points Φ p and Ψ p are at distance 0. The (quotient) metric space associated to this predistance is the desired space.

This is an instance of a more general construction, where Φ and Ψ do not have to be isometries, but the distances in the image almost coincide, up to say. Then one can almost glue the two spaces so that the images of a point under Φ and Ψ are ε-close. If ε > 0, this yields a metric space structure on X ⊕ Y, without the need to take a quotient. In particular, this gives a natural metric space structure on X ⊕ Y, where the basepoints are at distance 1, say, and the distances between other points are obtained by going through the two basepoints. (We also register the same metric space structure on a general disjoint union Σ i, E i).

We also define the inductive limit of metric spaces. Given

     f 0        f 1        f 2        f 3
X 0 -----> X 1 -----> X 2 -----> X 3 -----> ...

where the X n are metric spaces and f n isometric embeddings, we define the inductive limit of the X n, also known as the increasing union of the X n in this context, if we identify X n and X (n+1) through f n. This is a metric space in which all X n embed isometrically and in a way compatible with f n.

noncomputable def metric.glue_dist {X : Type u} {Y : Type v} {Z : Type w} [metric_space X] [metric_space Y] (Φ : Z X) (Ψ : Z Y) (ε : ) :
X Y X Y

Define a predistance on X ⊕ Y, for which Φ p and Ψ p are at distance ε

Equations
theorem metric.glue_dist_glued_points {X : Type u} {Y : Type v} {Z : Type w} [metric_space X] [metric_space Y] [nonempty Z] (Φ : Z X) (Ψ : Z Y) (ε : ) (p : Z) :
metric.glue_dist Φ Ψ ε (sum.inl (Φ p)) (sum.inr (Ψ p)) = ε
noncomputable def metric.glue_metric_approx {X : Type u} {Y : Type v} {Z : Type w} [metric_space X] [metric_space Y] [nonempty Z] (Φ : Z X) (Ψ : Z Y) (ε : ) (ε0 : 0 < ε) (H : (p q : Z), |has_dist.dist (Φ p) (Φ q) - has_dist.dist (Ψ p) (Ψ q)| 2 * ε) :

Given two maps Φ and Ψ intro metric spaces X and Y such that the distances between Φ p and Φ q, and between Ψ p and Ψ q, coincide up to 2 ε where ε > 0, one can almost glue the two spaces X and Y along the images of Φ and Ψ, so that Φ p and Ψ p are at distance ε.

Equations
noncomputable def metric.sum.dist {X : Type u} {Y : Type v} [metric_space X] [metric_space Y] :
X Y X Y

Distance on a disjoint union. There are many (noncanonical) ways to put a distance compatible with each factor. If the two spaces are bounded, one can say for instance that each point in the first is at distance diam X + diam Y + 1 of each point in the second. Instead, we choose a construction that works for unbounded spaces, but requires basepoints, chosen arbitrarily. We embed isometrically each factor, set the basepoints at distance 1, arbitrarily, and say that the distance from a to b is the sum of the distances of a and b to their respective basepoints, plus the distance 1 between the basepoints. Since there is an arbitrary choice in this construction, it is not an instance by default.

Equations
theorem metric.sum.dist_eq_glue_dist {X : Type u} {Y : Type v} [metric_space X] [metric_space Y] {p q : X Y} (x : X) (y : Y) :
metric.sum.dist p q = metric.glue_dist (λ (_x : unit), _.some) (λ (_x : unit), _.some) 1 p q
theorem metric.sum.one_dist_le {X : Type u} {Y : Type v} [metric_space X] [metric_space Y] {x : X} {y : Y} :
theorem metric.sum.one_dist_le' {X : Type u} {Y : Type v} [metric_space X] [metric_space Y] {x : X} {y : Y} :
noncomputable def metric.metric_space_sum {X : Type u} {Y : Type v} [metric_space X] [metric_space Y] :

The distance on the disjoint union indeed defines a metric space. All the distance properties follow from our choice of the distance. The harder work is to show that the uniform structure defined by the distance coincides with the disjoint union uniform structure.

Equations
theorem metric.sum.dist_eq {X : Type u} {Y : Type v} [metric_space X] [metric_space Y] {x y : X Y} :

The left injection of a space in a disjoint union is an isometry

The right injection of a space in a disjoint union is an isometry

@[protected]
noncomputable def metric.sigma.dist {ι : Type u_1} {E : ι Type u_2} [Π (i : ι), metric_space (E i)] :
(Σ (i : ι), E i) (Σ (i : ι), E i)

Distance on a disjoint union. There are many (noncanonical) ways to put a distance compatible with each factor. We choose a construction that works for unbounded spaces, but requires basepoints, chosen arbitrarily. We embed isometrically each factor, set the basepoints at distance 1, arbitrarily, and say that the distance from a to b is the sum of the distances of a and b to their respective basepoints, plus the distance 1 between the basepoints. Since there is an arbitrary choice in this construction, it is not an instance by default.

Equations
noncomputable def metric.sigma.has_dist {ι : Type u_1} {E : ι Type u_2} [Π (i : ι), metric_space (E i)] :
has_dist (Σ (i : ι), E i)

A has_dist instance on the disjoint union Σ i, E i. We embed isometrically each factor, set the basepoints at distance 1, arbitrarily, and say that the distance from a to b is the sum of the distances of a and b to their respective basepoints, plus the distance 1 between the basepoints. Since there is an arbitrary choice in this construction, it is not an instance by default.

Equations
@[simp]
theorem metric.sigma.dist_same {ι : Type u_1} {E : ι Type u_2} [Π (i : ι), metric_space (E i)] (i : ι) (x y : E i) :
has_dist.dist i, x⟩ i, y⟩ = has_dist.dist x y
@[simp]
theorem metric.sigma.dist_ne {ι : Type u_1} {E : ι Type u_2} [Π (i : ι), metric_space (E i)] {i j : ι} (h : i j) (x : E i) (y : E j) :
theorem metric.sigma.one_le_dist_of_ne {ι : Type u_1} {E : ι Type u_2} [Π (i : ι), metric_space (E i)] {i j : ι} (h : i j) (x : E i) (y : E j) :
1 has_dist.dist i, x⟩ j, y⟩
theorem metric.sigma.fst_eq_of_dist_lt_one {ι : Type u_1} {E : ι Type u_2} [Π (i : ι), metric_space (E i)] (x y : Σ (i : ι), E i) (h : has_dist.dist x y < 1) :
x.fst = y.fst
@[protected]
theorem metric.sigma.dist_triangle {ι : Type u_1} {E : ι Type u_2} [Π (i : ι), metric_space (E i)] (x y z : Σ (i : ι), E i) :
@[protected]
theorem metric.sigma.is_open_iff {ι : Type u_1} {E : ι Type u_2} [Π (i : ι), metric_space (E i)] (s : set (Σ (i : ι), E i)) :
is_open s (x : Σ (i : ι), E i), x s ( (ε : ) (H : ε > 0), (y : Σ (i : ι), E i), has_dist.dist x y < ε y s)
@[protected]
noncomputable def metric.sigma.metric_space {ι : Type u_1} {E : ι Type u_2} [Π (i : ι), metric_space (E i)] :
metric_space (Σ (i : ι), E i)

A metric space structure on the disjoint union Σ i, E i. We embed isometrically each factor, set the basepoints at distance 1, arbitrarily, and say that the distance from a to b is the sum of the distances of a and b to their respective basepoints, plus the distance 1 between the basepoints. Since there is an arbitrary choice in this construction, it is not an instance by default.

Equations
theorem metric.sigma.isometry_mk {ι : Type u_1} {E : ι Type u_2} [Π (i : ι), metric_space (E i)] (i : ι) :

The injection of a space in a disjoint union is an isometry

@[protected]
theorem metric.sigma.complete_space {ι : Type u_1} {E : ι Type u_2} [Π (i : ι), metric_space (E i)] [ (i : ι), complete_space (E i)] :
complete_space (Σ (i : ι), E i)

A disjoint union of complete metric spaces is complete.

noncomputable def metric.glue_premetric {X : Type u} {Y : Type v} {Z : Type w} [nonempty Z] [metric_space Z] [metric_space X] [metric_space Y] {Φ : Z X} {Ψ : Z Y} (hΦ : isometry Φ) (hΨ : isometry Ψ) :

Given two isometric embeddings Φ : Z → X and Ψ : Z → Y, we define a pseudo metric space structure on X ⊕ Y by declaring that Φ x and Ψ x are at distance 0.

Equations
@[protected, instance]
noncomputable def metric.glue_space.metric_space {X : Type u} {Y : Type v} {Z : Type w} [nonempty Z] [metric_space Z] [metric_space X] [metric_space Y] {Φ : Z X} {Ψ : Z Y} (hΦ : isometry Φ) (hΨ : isometry Ψ) :
def metric.glue_space {X : Type u} {Y : Type v} {Z : Type w} [nonempty Z] [metric_space Z] [metric_space X] [metric_space Y] {Φ : Z X} {Ψ : Z Y} (hΦ : isometry Φ) (hΨ : isometry Ψ) :
Type (max u v)

Given two isometric embeddings Φ : Z → X and Ψ : Z → Y, we define a space glue_space hΦ hΨ by identifying in X ⊕ Y the points Φ x and Ψ x.

Equations
Instances for metric.glue_space
noncomputable def metric.to_glue_l {X : Type u} {Y : Type v} {Z : Type w} [nonempty Z] [metric_space Z] [metric_space X] [metric_space Y] {Φ : Z X} {Ψ : Z Y} (hΦ : isometry Φ) (hΨ : isometry Ψ) (x : X) :

The canonical map from X to the space obtained by gluing isometric subsets in X and Y.

Equations
noncomputable def metric.to_glue_r {X : Type u} {Y : Type v} {Z : Type w} [nonempty Z] [metric_space Z] [metric_space X] [metric_space Y] {Φ : Z X} {Ψ : Z Y} (hΦ : isometry Φ) (hΨ : isometry Ψ) (y : Y) :

The canonical map from Y to the space obtained by gluing isometric subsets in X and Y.

Equations
@[protected, instance]
noncomputable def metric.inhabited_left {X : Type u} {Y : Type v} {Z : Type w} [nonempty Z] [metric_space Z] [metric_space X] [metric_space Y] {Φ : Z X} {Ψ : Z Y} (hΦ : isometry Φ) (hΨ : isometry Ψ) [inhabited X] :
Equations
@[protected, instance]
noncomputable def metric.inhabited_right {X : Type u} {Y : Type v} {Z : Type w} [nonempty Z] [metric_space Z] [metric_space X] [metric_space Y] {Φ : Z X} {Ψ : Z Y} (hΦ : isometry Φ) (hΨ : isometry Ψ) [inhabited Y] :
Equations
theorem metric.to_glue_commute {X : Type u} {Y : Type v} {Z : Type w} [nonempty Z] [metric_space Z] [metric_space X] [metric_space Y] {Φ : Z X} {Ψ : Z Y} (hΦ : isometry Φ) (hΨ : isometry Ψ) :
metric.to_glue_l Φ = metric.to_glue_r Ψ
theorem metric.to_glue_l_isometry {X : Type u} {Y : Type v} {Z : Type w} [nonempty Z] [metric_space Z] [metric_space X] [metric_space Y] {Φ : Z X} {Ψ : Z Y} (hΦ : isometry Φ) (hΨ : isometry Ψ) :
theorem metric.to_glue_r_isometry {X : Type u} {Y : Type v} {Z : Type w} [nonempty Z] [metric_space Z] [metric_space X] [metric_space Y] {Φ : Z X} {Ψ : Z Y} (hΦ : isometry Φ) (hΨ : isometry Ψ) :
def metric.inductive_limit_dist {X : Type u} [Π (n : ), metric_space (X n)] (f : Π (n : ), X n X (n + 1)) (x y : Σ (n : ), X n) :

Predistance on the disjoint union Σ n, X n.

Equations
theorem metric.inductive_limit_dist_eq_dist {X : Type u} [Π (n : ), metric_space (X n)] {f : Π (n : ), X n X (n + 1)} (I : (n : ), isometry (f n)) (x y : Σ (n : ), X n) (m : ) (hx : x.fst m) (hy : y.fst m) :

The predistance on the disjoint union Σ n, X n can be computed in any X k for large enough k.

def metric.inductive_premetric {X : Type u} [Π (n : ), metric_space (X n)] {f : Π (n : ), X n X (n + 1)} (I : (n : ), isometry (f n)) :

Premetric space structure on Σ n, X n.

Equations
@[protected, instance]
def metric.inductive_limit.metric_space {X : Type u} [Π (n : ), metric_space (X n)] {f : Π (n : ), X n X (n + 1)} (I : (n : ), isometry (f n)) :
def metric.inductive_limit {X : Type u} [Π (n : ), metric_space (X n)] {f : Π (n : ), X n X (n + 1)} (I : (n : ), isometry (f n)) :

The type giving the inductive limit in a metric space context.

Equations
Instances for metric.inductive_limit
def metric.to_inductive_limit {X : Type u} [Π (n : ), metric_space (X n)] {f : Π (n : ), X n X (n + 1)} (I : (n : ), isometry (f n)) (n : ) (x : X n) :

Mapping each X n to the inductive limit.

Equations
@[protected, instance]
def metric.inductive_limit.inhabited {X : Type u} [Π (n : ), metric_space (X n)] {f : Π (n : ), X n X (n + 1)} (I : (n : ), isometry (f n)) [inhabited (X 0)] :
Equations
theorem metric.to_inductive_limit_isometry {X : Type u} [Π (n : ), metric_space (X n)] {f : Π (n : ), X n X (n + 1)} (I : (n : ), isometry (f n)) (n : ) :

The map to_inductive_limit n mapping X n to the inductive limit is an isometry.

theorem metric.to_inductive_limit_commute {X : Type u} [Π (n : ), metric_space (X n)] {f : Π (n : ), X n X (n + 1)} (I : (n : ), isometry (f n)) (n : ) :

The maps to_inductive_limit n are compatible with the maps f n.