This repository was archived by the owner on Jul 24, 2024. It is now read-only.
File tree Expand file tree Collapse file tree 1 file changed +6
-2
lines changed Expand file tree Collapse file tree 1 file changed +6
-2
lines changed Original file line number Diff line number Diff line change 83
83
section Profinite
84
84
local attribute [instance] connected_component_setoid
85
85
86
+ universes u
87
+
86
88
/--
87
89
(Implementation) The object part of the connected_components functor from compact Hausdorff spaces
88
90
to Profinite spaces, given by quotienting a space by its connected components.
89
91
See: https://stacks.math.columbia.edu/tag/0900
90
92
-/
91
- def CompHaus.to_Profinite_obj (X : CompHaus) : Profinite :=
93
+ -- Without explicit universe annotations here, Lean introduces two universe variables and
94
+ -- unhelpfully defines a function `CompHaus.{max u₁ u₂} → Profinite.{max u₁ u₂}`.
95
+ def CompHaus.to_Profinite_obj (X : CompHaus.{u}) : Profinite.{u} :=
92
96
{ to_Top := { α := connected_components X.to_Top.α },
93
97
is_compact := quotient.compact_space,
94
98
is_t2 := connected_components.t2,
@@ -98,7 +102,7 @@ def CompHaus.to_Profinite_obj (X : CompHaus) : Profinite :=
98
102
(Implementation) The bijection of homsets to establish the reflective adjunction of Profinite
99
103
spaces in compact Hausdorff spaces.
100
104
-/
101
- def Profinite.to_CompHaus_equivalence (X : CompHaus) (Y : Profinite) :
105
+ def Profinite.to_CompHaus_equivalence (X : CompHaus.{u} ) (Y : Profinite.{u} ) :
102
106
(CompHaus.to_Profinite_obj X ⟶ Y) ≃ (X ⟶ Profinite.to_CompHaus.obj Y) :=
103
107
{ to_fun := λ f,
104
108
{ to_fun := f.1 ∘ quotient.mk,
You can’t perform that action at this time.
0 commit comments