Skip to content

Commit e9eb901

Browse files
committed
chore: reorder universes in ConcreteCategory (#5605)
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
1 parent 4d4f0f2 commit e9eb901

File tree

2 files changed

+9
-9
lines changed

2 files changed

+9
-9
lines changed

Mathlib/AlgebraicGeometry/AffineScheme.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -630,7 +630,7 @@ theorem IsAffineOpen.isLocalization_stalk_aux {X : Scheme} (U : Opens X)
630630
rw [eqToHom_trans]
631631
#align algebraic_geometry.is_affine_open.is_localization_stalk_aux AlgebraicGeometry.IsAffineOpen.isLocalization_stalk_aux
632632

633-
set_option maxHeartbeats 1643256 in
633+
set_option maxHeartbeats 3200000 in
634634
theorem IsAffineOpen.isLocalization_stalk_aux' {X : Scheme} {U : Opens X} (hU : IsAffineOpen U)
635635
(y : PrimeSpectrum (X.presheaf.obj <| op U)) (hy : hU.fromSpec.1.base y ∈ U) :
636636
hU.fromSpec.val.c.app (op U) ≫ (Scheme.Spec.obj <| op (X.presheaf.obj <| op U)).presheaf.germ
@@ -661,7 +661,7 @@ theorem IsAffineOpen.isLocalization_stalk_aux' {X : Scheme} {U : Opens X} (hU :
661661
rw [Category.id_comp]
662662
rfl
663663

664-
set_option maxHeartbeats 420000 in
664+
set_option maxHeartbeats 800000 in
665665
theorem IsAffineOpen.isLocalization_stalk' {X : Scheme} {U : Opens X} (hU : IsAffineOpen U)
666666
(y : PrimeSpectrum (X.presheaf.obj <| op U)) (hy : hU.fromSpec.1.base y ∈ U) :
667667
haveI : IsAffine _ := hU

Mathlib/CategoryTheory/ConcreteCategory/Basic.lean

Lines changed: 7 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Scott Morrison, Johannes Hölzl, Reid Barton, Sean Leather, Yury Kudryashov
55
66
! This file was ported from Lean 3 source module category_theory.concrete_category.basic
7-
! leanprover-community/mathlib commit 05b820ec79b3c98a7dbf1cb32e181584166da2ca
7+
! leanprover-community/mathlib commit 311ef8c4b4ae2804ea76b8a611bc5ea1d9c16872
88
! Please do not edit these lines, except to modify the commit id
99
! if you have ported upstream changes.
1010
-/
@@ -41,7 +41,7 @@ related work.
4141
-/
4242

4343

44-
universe w w' v v' u
44+
universe w w' v v' u u'
4545

4646
namespace CategoryTheory
4747

@@ -68,13 +68,13 @@ attribute [instance] ConcreteCategory.forget_faithful
6868

6969
/-- The forgetful functor from a concrete category to `Type u`. -/
7070
@[reducible]
71-
def forget (C : Type v) [Category C] [ConcreteCategory.{u} C] : C ⥤ Type u :=
71+
def forget (C : Type u) [Category.{v} C] [ConcreteCategory.{w} C] : C ⥤ Type w :=
7272
ConcreteCategory.forget
7373
#align category_theory.forget CategoryTheory.forget
7474

7575
-- this is reducible because we want `forget (Type u)` to unfold to `𝟭 _`
7676
@[reducible]
77-
instance ConcreteCategory.types : ConcreteCategory (Type u) where
77+
instance ConcreteCategory.types : ConcreteCategory.{u, u, u+1} (Type u) where
7878
forget := 𝟭 _
7979
#align category_theory.concrete_category.types CategoryTheory.ConcreteCategory.types
8080

@@ -86,16 +86,16 @@ You can use it on particular examples as:
8686
instance : HasCoeToSort X := ConcreteCategory.hasCoeToSort X
8787
```
8888
-/
89-
def ConcreteCategory.hasCoeToSort (C : Type v) [Category C] [ConcreteCategory C] :
90-
CoeSort C (Type u) where
89+
def ConcreteCategory.hasCoeToSort (C : Type u) [Category.{v} C] [ConcreteCategory.{w} C] :
90+
CoeSort C (Type w) where
9191
coe := fun X => (forget C).obj X
9292
#align category_theory.concrete_category.has_coe_to_sort CategoryTheory.ConcreteCategory.hasCoeToSort
9393

9494
section
9595

9696
attribute [local instance] ConcreteCategory.hasCoeToSort
9797

98-
variable {C : Type v} [Category C] [ConcreteCategory.{w} C]
98+
variable {C : Type u} [Category.{v} C] [ConcreteCategory.{w} C]
9999

100100
-- Porting note: forget_obj_eq_coe has become a syntactic tautology.
101101
#noalign category_theory.forget_obj_eq_coe

0 commit comments

Comments
 (0)