The category of Profinite Types #
We construct the category of profinite topological spaces, often called profinite sets -- perhaps they could be called profinite types in Lean.
The type of profinite topological spaces is called Profinite
. It has a category
instance and is a fully faithful subcategory of Top
. The fully faithful functor
is called Profinite_to_Top
.
Implementation notes #
A profinite type is defined to be a topological space which is compact, Hausdorff and totally disconnected.
TODO #
- Link to category of projective limits of finite discrete sets.
- existence of products, limits(?), finite coproducts
Profinite_to_Top
creates limits?- Clausen/Scholze topology on the category
Profinite
.
Tags #
profinite
Equations
- Profinite.inhabited = {default := {to_Top := {α := pempty, str := pempty.topological_space}, is_compact := Profinite.inhabited._proof_1, is_t2 := Profinite.inhabited._proof_2, is_totally_disconnected := Profinite.inhabited._proof_3}}
Equations
- Profinite.to_CompHaus.category_theory.full = {preimage := λ (_x _x_1 : Profinite) (f : Profinite.to_CompHaus.obj _x ⟶ Profinite.to_CompHaus.obj _x_1), f, witness' := Profinite.to_CompHaus.category_theory.full._proof_1}
(Implementation) The object part of the connected_components functor from compact Hausdorff spaces to Profinite spaces, given by quotienting a space by its connected components. See: https://stacks.math.columbia.edu/tag/0900
Equations
- X.to_Profinite_obj = Profinite.mk {α := connected_components X.to_Top.α X.to_Top.topological_space, str := {is_open := λ (s : set (quotient (connected_component_setoid X.to_Top.α))), X.to_Top.topological_space.is_open (quotient.mk ⁻¹' s), is_open_univ := _, is_open_inter := _, is_open_sUnion := _}}
(Implementation) The bijection of homsets to establish the reflective adjunction of Profinite spaces in compact Hausdorff spaces.
Equations
- Profinite.to_CompHaus_equivalence X Y = {to_fun := λ (f : X.to_Profinite_obj ⟶ Y), {to_fun := f.to_fun ∘ quotient.mk, continuous_to_fun := _}, inv_fun := λ (g : X ⟶ Profinite.to_CompHaus.obj Y), {to_fun := continuous.connected_components_lift _, continuous_to_fun := _}, left_inv := _, right_inv := _}
The connected_components functor from compact Hausdorff spaces to profinite spaces, left adjoint to the inclusion functor.
Equations
- CompHaus.to_Profinite = category_theory.adjunction.left_adjoint_of_equiv Profinite.to_CompHaus_equivalence CompHaus.to_Profinite._proof_1
The adjunction between CompHaus.to_Profinite and Profinite.to_CompHaus
Equations
- Profinite.to_Profinite_adj_to_CompHaus = category_theory.adjunction.adjunction_of_equiv_left Profinite.to_CompHaus_equivalence CompHaus.to_Profinite._proof_1
The category of profinite sets is reflective in the category of compact hausdroff spaces