Profinite sets as limits of finite sets. #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We show that any profinite set is isomorphic to the limit of its discrete (hence finite) quotients.
Definitions #
There are a handful of definitions in this file, given X : Profinite
:
X.fintype_diagram
is the functordiscrete_quotient X ⥤ Fintype
whose limit is isomorphic toX
(the limit taking place inProfinite
viaFintype_to_Profinite
, see 2).X.diagram
is an abbreviation forX.fintype_diagram ⋙ Fintype_to_Profinite
.X.as_limit_cone
is the cone overX.diagram
whose cone point isX
.X.iso_as_limit_cone_lift
is the isomorphismX ≅ (Profinite.limit_cone X.diagram).X
induced by liftingX.as_limit_cone
.X.as_limit_cone_iso
is the isomorphismX.as_limit_cone ≅ (Profinite.limit_cone X.diagram)
induced byX.iso_as_limit_cone_lift
.X.as_limit
is a term of typeis_limit X.as_limit_cone
.X.lim : category_theory.limits.limit_cone X.as_limit_cone
is a bundled combination of 3 and 6.
The functor discrete_quotient X ⥤ Fintype
whose limit is isomorphic to X
.
Equations
- X.fintype_diagram = {obj := λ (S : discrete_quotient ↥X), Fintype.of ↥S, map := λ (S T : discrete_quotient ↥X) (f : S ⟶ T), discrete_quotient.of_le _, map_id' := _, map_comp' := _}
An abbreviation for X.fintype_diagram ⋙ Fintype_to_Profinite
.
A cone over X.diagram
whose cone point is X
.
Equations
- X.as_limit_cone = {X := X, π := {app := λ (S : discrete_quotient ↥X), {to_fun := S.proj, continuous_to_fun := _}, naturality' := _}}
The isomorphism between X
and the explicit limit of X.diagram
,
induced by lifting X.as_limit_cone
.
Equations
The isomorphism of cones X.as_limit_cone
and Profinite.limit_cone X.diagram
.
The underlying isomorphism is defeq to X.iso_as_limit_cone_lift
.
X.as_limit_cone
is indeed a limit cone.
Equations
A bundled version of X.as_limit_cone
and X.as_limit
.