Documentation

Mathlib.Topology.UniformSpace.Closeds

Hausdorff uniformity #

This file defines the Hausdorff uniformity on the types of closed subsets, compact subsets and and nonempty compact subsets of a uniform space. This is the generalization of the uniformity induced by the Hausdorff metric to hyperspaces of uniform spaces.

def hausdorffEntourage {α : Type u_1} (U : SetRel α α) :
SetRel (Set α) (Set α)

The set of pairs of sets contained in each other's thickening with respect to an entourage.

Equations
Instances For
    theorem mem_hausdorffEntourage {α : Type u_1} (U : SetRel α α) (s t : Set α) :
    theorem hausdorffEntourage_mono {α : Type u_1} {U V : SetRel α α} (h : U V) :
    @[simp]
    theorem singleton_mem_hausdorffEntourage {α : Type u_1} (U : SetRel α α) (x y : α) :
    @[reducible, inline]

    The Hausdorff uniformity on the powerset of a uniform space. Used for defining the uniformities on Closeds, Compacts and NonemptyCompacts. See note [reducible non-instances].

    Equations
    Instances For
      theorem Filter.HasBasis.uniformity_hausdorff {α : Type u_1} [UniformSpace α] {ι : Sort u_2} {p : ιProp} {s : ιSet (α × α)} (h : (uniformity α).HasBasis p s) :

      In the Hausdorff uniformity, the powerset of a totally bounded set is totally bounded.

      theorem Filter.HasBasis.uniformity_closeds {α : Type u_1} [UniformSpace α] {ι : Sort u_2} {p : ιProp} {s : ιSet (α × α)} (h : (uniformity α).HasBasis p s) :
      theorem Filter.HasBasis.uniformity_compacts {α : Type u_1} [UniformSpace α] {ι : Sort u_2} {p : ιProp} {s : ιSet (α × α)} (h : (uniformity α).HasBasis p s) :