The set of functions on α ⊕ β that are candidates distances to realize the minimum of the Hausdorff distances between α and β in a coupling
Equations
- Gromov_Hausdorff.candidates α β = {f : prod_space_fun α β | (((((∀ (x y : α), f (sum.inl x, sum.inl y) = has_dist.dist x y) ∧ ∀ (x y : β), f (sum.inr x, sum.inr y) = has_dist.dist x y) ∧ ∀ (x y : α ⊕ β), f (x, y) = f (y, x)) ∧ ∀ (x y z : α ⊕ β), f (x, z) ≤ f (x, y) + f (y, z)) ∧ ∀ (x : α ⊕ β), f (x, x) = 0) ∧ ∀ (x y : α ⊕ β), f (x, y) ≤ ↑(max_var α β)}
candidates give rise to elements of bounded_continuous_functions
Equations
- Gromov_Hausdorff.candidates_b_dist α β = Gromov_Hausdorff.candidates_b_of_candidates (λ (p : (α ⊕ β) × (α ⊕ β)), has_dist.dist p.fst p.snd) _
We will then choose the candidate minimizing the Hausdorff distance. Except that we are not in a metric space setting, so we need to define our custom version of Hausdorff distance, called HD, and prove its basic properties.
Explicit bound on HD (dist). This means that when looking for minimizers it will be sufficient to look for functions with HD(f) bounded by this bound.
With the optimal candidate, construct a premetric space structure on α ⊕ β, on which the predistance is given by the candidate. Then, we will identify points at 0 predistance to obtain a genuine metric space
Equations
- Gromov_Hausdorff.premetric_optimal_GH_dist α β = {to_has_dist := {dist := λ (p q : α ⊕ β), ⇑(optimal_GH_dist α β) (p, q)}, dist_self := _, dist_comm := _, dist_triangle := _}
A metric space which realizes the optimal coupling between α and β
Equations
Injection of α in the optimal coupling between α and β
Equations
The injection of α in the optimal coupling between α and β is an isometry.
Injection of β in the optimal coupling between α and β
Equations
The injection of β in the optimal coupling between α and β is an isometry.
The optimal coupling between two compact spaces α and β is still a compact space
Equations
- _ = _
For any candidate f, HD(f) is larger than or equal to the Hausdorff distance in the optimal coupling. This follows from the fact that HD of the optimal candidate is exactly the Hausdorff distance in the optimal coupling, although we only prove here the inequality we need.