mathlib documentation

topology.​uniform_space.​separation

topology.​uniform_space.​separation

Hausdorff properties of uniform spaces. Separation quotient.

This file studies uniform spaces whose underlying topological spaces are separated (also known as Hausdorff or T₂). This turns out to be equivalent to asking that the intersection of all entourages is the diagonal only. This condition actually implies the stronger separation property that the space is regular (T₃), hence those conditions are equivalent for topologies coming from a uniform structure.

More generally, the intersection 𝓢 X of all entourages of X, which has type set (X × X) is an equivalence relation on X. Points which are equivalent under the relation are basically undistinguishable from the point of view of the uniform structure. For instance any uniformly continuous function will send equivalent points to the same value.

The quotient separation_quotient X of X by 𝓢 X has a natural uniform structure which is separated, and satisfies a universal property: every uniformly continuous function from X to a separated uniform space uniquely factors through separation_quotient X. As usual, this allows to turn separation_quotient into a functor (but we don't use the category theory library in this file).

These notions admit relative versions, one can ask that s : set X is separated, this is equivalent to asking that the uniform structure induced on s is separated.

Main definitions

Main results

 Notations

Localized in uniformity, we have the notation 𝓢 X for the separation relation on a uniform space X,

Implementation notes

The separation setoid separation_setoid is not declared as a global instance. It is made a local instance while building the theory of separation_quotient. The factored map separation_quotient.lift f is defined without imposing any condition on f, but returns junk if f is not uniformly continuous (constant junk hence it is always uniformly continuous).

Separated uniform spaces

def separation_rel (α : Type u) [u : uniform_space α] :
set × α)

The separation relation is the intersection of all entourages. Two points which are related by the separation relation are "indistinguishable" according to the uniform structure.

Equations
theorem separated_equiv {α : Type u} [uniform_space α] :
equivalence (λ (x y : α), (x, y) separation_rel α)

theorem separated_def {α : Type u} [uniform_space α] :
separated_space α ∀ (x y : α), (∀ (r : set × α)), r uniformity α(x, y) r)x = y

theorem separated_def' {α : Type u} [uniform_space α] :
separated_space α ∀ (x y : α), x y(∃ (r : set × α)) (H : r uniformity α), (x, y) r)

theorem separation_rel_comap {α : Type u} {β : Type v} [uniform_space α] [uniform_space β] {f : α → β} :

theorem filter.​has_basis.​separation_rel {α : Type u} [uniform_space α] {ι : Type u_1} {p : ι → Prop} {s : ι → set × α)} :
(uniformity α).has_basis p s(separation_rel α = ⋂ (i : ι) (H : i set_of p), s i)

theorem separated_iff_t2 {α : Type u} [uniform_space α] :

@[instance]
def separated_regular {α : Type u} [uniform_space α] [separated_space α] :

Equations

 Separated sets

def is_separated {α : Type u} [uniform_space α] :
set α → Prop

A set s in a uniform space α is separated if the separation relation 𝓢 α induces the trivial relation on s.

Equations
theorem is_separated_def {α : Type u} [uniform_space α] (s : set α) :
is_separated s ∀ (x y : α), x sy s(x, y) separation_rel αx = y

theorem is_separated_def' {α : Type u} [uniform_space α] (s : set α) :

theorem eq_of_uniformity_inf_nhds_of_is_separated {α : Type u} [uniform_space α] {s : set α} (hs : is_separated s) {x y : α} :
x sy scluster_pt (x, y) (uniformity α)x = y

theorem eq_of_uniformity_inf_nhds {α : Type u} [uniform_space α] [separated_space α] {x y : α} :
cluster_pt (x, y) (uniformity α)x = y

Separation quotient

The separation relation of a uniform space seen as a setoid.

Equations
theorem uniform_space.​uniform_continuous_quotient_lift {α : Type u} {β : Type v} [uniform_space α] [uniform_space β] {f : α → β} {h : ∀ (a b : α), (a, b) separation_rel αf a = f b} :

theorem uniform_space.​uniform_continuous_quotient_lift₂ {α : Type u} {β : Type v} {γ : Type w} [uniform_space α] [uniform_space β] [uniform_space γ] {f : α → β → γ} {h : ∀ (a : α) (c : β) (b : α) (d : β), (a, b) separation_rel α(c, d) separation_rel βf a c = f b d} :

theorem uniform_space.​separated_of_uniform_continuous {α : Type u} {β : Type v} [uniform_space α] [uniform_space β] {f : α → β} {x y : α} :
uniform_continuous fx yf x f y

theorem uniform_space.​eq_of_separated_of_uniform_continuous {α : Type u} {β : Type v} [uniform_space α] [uniform_space β] [separated_space β] {f : α → β} {x y : α} :
uniform_continuous fx yf x = f y

def uniform_space.​separation_quotient (α : Type u_1) [uniform_space α] :
Type u_1

The maximal separated quotient of a uniform space α.

Equations
def uniform_space.​separation_quotient.​lift {α : Type u} {β : Type v} [uniform_space α] [uniform_space β] [separated_space β] :
(α → β)uniform_space.separation_quotient α → β

Factoring functions to a separated space through the separation quotient.

Equations
theorem uniform_space.​separation_quotient.​map_mk {α : Type u} {β : Type v} [uniform_space α] [uniform_space β] {f : α → β} (h : uniform_continuous f) (a : α) :

theorem uniform_space.​separation_prod {α : Type u} {β : Type v} [uniform_space α] [uniform_space β] {a₁ a₂ : α} {b₁ b₂ : β} :
(a₁, b₁) (a₂, b₂) a₁ a₂ b₁ b₂

@[instance]

Equations