Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit a0e2b3c

Browse files
committed
chore(topology/Profinite): reduce universe variables (#6300)
See https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/universe.20issue Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
1 parent 64d86f7 commit a0e2b3c

File tree

1 file changed

+6
-2
lines changed

1 file changed

+6
-2
lines changed

src/topology/category/Profinite.lean

Lines changed: 6 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -83,12 +83,16 @@ rfl
8383
section Profinite
8484
local attribute [instance] connected_component_setoid
8585

86+
universes u
87+
8688
/--
8789
(Implementation) The object part of the connected_components functor from compact Hausdorff spaces
8890
to Profinite spaces, given by quotienting a space by its connected components.
8991
See: https://stacks.math.columbia.edu/tag/0900
9092
-/
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} :=
9296
{ to_Top := { α := connected_components X.to_Top.α },
9397
is_compact := quotient.compact_space,
9498
is_t2 := connected_components.t2,
@@ -98,7 +102,7 @@ def CompHaus.to_Profinite_obj (X : CompHaus) : Profinite :=
98102
(Implementation) The bijection of homsets to establish the reflective adjunction of Profinite
99103
spaces in compact Hausdorff spaces.
100104
-/
101-
def Profinite.to_CompHaus_equivalence (X : CompHaus) (Y : Profinite) :
105+
def Profinite.to_CompHaus_equivalence (X : CompHaus.{u}) (Y : Profinite.{u}) :
102106
(CompHaus.to_Profinite_obj X ⟶ Y) ≃ (X ⟶ Profinite.to_CompHaus.obj Y) :=
103107
{ to_fun := λ f,
104108
{ to_fun := f.1 ∘ quotient.mk,

0 commit comments

Comments
 (0)