mathlib3 documentation

topology.discrete_quotient

Discrete quotients of a topological space. #

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

This file defines the type of discrete quotients of a topological space, denoted discrete_quotient X. To avoid quantifying over types, we model such quotients as setoids whose equivalence classes are clopen.

Definitions #

  1. discrete_quotient X is the type of discrete quotients of X. It is endowed with a coercion to Type, which is defined as the quotient associated to the setoid in question, and each such quotient is endowed with the discrete topology.
  2. Given S : discrete_quotient X, the projection X → S is denoted S.proj.
  3. When X is compact and S : discrete_quotient X, the space S is endowed with a fintype instance.

Order structure #

The type discrete_quotient X is endowed with an instance of a semilattice_inf with order_top. The partial ordering A ≤ B mathematically means that B.proj factors through A.proj. The top element is the trivial quotient, meaning that every element of X is collapsed to a point. Given h : A ≤ B, the map A → B is discrete_quotient.of_le h.

Whenever X is a locally connected space, the type discrete_quotient X is also endowed with an instance of a order_bot, where the bot element is given by the connectedComponentSetoid, i.e., x ~ y means that x and y belong to the same connected component. In particular, if X is a discrete topological space, then x ~ y is equivalent (propositionally, not definitionally) to x = y.

Given f : C(X, Y), we define a predicate discrete_quotient.le_comap f A B for A : discrete_quotient X and B : discrete_quotient Y, asserting that f descends to A → B. If cond : discrete_quotient.le_comap h A B, the function A → B is obtained by discrete_quotient.map f cond.

Theorems #

The two main results proved in this file are:

  1. discrete_quotient.eq_of_forall_proj_eq which states that when X is compact, T₂, and totally disconnected, any two elements of X are equal if their projections in Q agree for all Q : discrete_quotient X.

  2. discrete_quotient.exists_of_compat which states that when X is compact, then any system of elements of Q as Q : discrete_quotient X varies, which is compatible with respect to discrete_quotient.of_le, must arise from some element of X.

Remarks #

The constructions in this file will be used to show that any profinite space is a limit of finite discrete spaces.

@[ext]
structure discrete_quotient (X : Type u_5) [topological_space X] :
Type u_5

The type of discrete quotients of a topological space.

Instances for discrete_quotient
theorem discrete_quotient.ext_iff {X : Type u_5} {_inst_4 : topological_space X} (x y : discrete_quotient X) :
theorem discrete_quotient.ext {X : Type u_5} {_inst_4 : topological_space X} (x y : discrete_quotient X) (h : x.to_setoid = y.to_setoid) :
x = y

Construct a discrete quotient from a clopen set.

Equations
theorem discrete_quotient.refl {X : Type u_2} [topological_space X] (S : discrete_quotient X) (x : X) :
theorem discrete_quotient.symm {X : Type u_2} [topological_space X] (S : discrete_quotient X) {x y : X} :
theorem discrete_quotient.trans {X : Type u_2} [topological_space X] (S : discrete_quotient X) {x y z : X} :

The projection from X to the given discrete quotient.

Equations
@[protected, instance]
Equations
@[protected, instance]

Comap a discrete quotient along a continuous map.

Equations
def discrete_quotient.of_le {X : Type u_2} [topological_space X] {A B : discrete_quotient X} (h : A B) :

The map induced by a refinement of a discrete quotient.

Equations
@[simp]
theorem discrete_quotient.of_le_of_le {X : Type u_2} [topological_space X] {A B C : discrete_quotient X} (h₁ : A B) (h₂ : B C) (x : A) :
@[simp]
theorem discrete_quotient.of_le_proj {X : Type u_2} [topological_space X] {A B : discrete_quotient X} (h : A B) (x : X) :
@[protected, instance]

When X is a locally connected space, there is an order_bot instance on discrete_quotient X. The bottom element is given by connected_component_setoid X

Equations
def discrete_quotient.le_comap {X : Type u_2} {Y : Type u_3} [topological_space X] [topological_space Y] (f : C(X, Y)) (A : discrete_quotient X) (B : discrete_quotient Y) :
Prop

Given f : C(X, Y), le_comap cont A B is defined as A ≤ B.comap f. Mathematically this means that f descends to a morphism A → B.

Equations
theorem discrete_quotient.le_comap.mono {X : Type u_2} {Y : Type u_3} [topological_space X] [topological_space Y] {f : C(X, Y)} {A A' : discrete_quotient X} {B B' : discrete_quotient Y} (h : discrete_quotient.le_comap f A B) (hA : A' A) (hB : B B') :

Map a discrete quotient along a continuous map.

Equations
@[simp]
theorem discrete_quotient.map_proj {X : Type u_2} {Y : Type u_3} [topological_space X] [topological_space Y] {f : C(X, Y)} {A : discrete_quotient X} {B : discrete_quotient Y} (cond : discrete_quotient.le_comap f A B) (x : X) :
discrete_quotient.map f cond (A.proj x) = B.proj (f x)
@[simp]
@[simp]
theorem discrete_quotient.eq_of_forall_proj_eq {X : Type u_2} [topological_space X] [t2_space X] [compact_space X] [disc : totally_disconnected_space X] {x y : X} (h : (Q : discrete_quotient X), Q.proj x = Q.proj y) :
x = y
theorem discrete_quotient.exists_of_compat {X : Type u_2} [topological_space X] [compact_space X] (Qs : Π (Q : discrete_quotient X), Q) (compat : (A B : discrete_quotient X) (h : A B), discrete_quotient.of_le h (Qs A) = Qs B) :
(x : X), (Q : discrete_quotient X), Q.proj x = Qs Q
@[protected, instance]

Any locally constant function induces a discrete quotient.

Equations

The (locally constant) function from the discrete quotient associated to a locally constant function.

Equations