@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
4
4
Authors: Scott Morrison, Johannes Hölzl, Reid Barton, Sean Leather, Yury Kudryashov
5
5
6
6
! 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
8
8
! Please do not edit these lines, except to modify the commit id
9
9
! if you have ported upstream changes.
10
10
-/
@@ -41,7 +41,7 @@ related work.
41
41
-/
42
42
43
43
44
- universe w w' v v' u
44
+ universe w w' v v' u u'
45
45
46
46
namespace CategoryTheory
47
47
@@ -68,13 +68,13 @@ attribute [instance] ConcreteCategory.forget_faithful
68
68
69
69
/-- The forgetful functor from a concrete category to `Type u`. -/
70
70
@[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 :=
72
72
ConcreteCategory.forget
73
73
#align category_theory.forget CategoryTheory.forget
74
74
75
75
-- this is reducible because we want `forget (Type u)` to unfold to `𝟭 _`
76
76
@[reducible]
77
- instance ConcreteCategory.types : ConcreteCategory (Type u) where
77
+ instance ConcreteCategory.types : ConcreteCategory.{u, u, u+ 1 } (Type u) where
78
78
forget := 𝟭 _
79
79
#align category_theory.concrete_category.types CategoryTheory.ConcreteCategory.types
80
80
@@ -86,16 +86,16 @@ You can use it on particular examples as:
86
86
instance : HasCoeToSort X := ConcreteCategory.hasCoeToSort X
87
87
```
88
88
-/
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
91
91
coe := fun X => (forget C).obj X
92
92
#align category_theory.concrete_category.has_coe_to_sort CategoryTheory.ConcreteCategory.hasCoeToSort
93
93
94
94
section
95
95
96
96
attribute [local instance] ConcreteCategory.hasCoeToSort
97
97
98
- variable {C : Type v } [Category C] [ConcreteCategory.{w} C]
98
+ variable {C : Type u } [Category.{v} C] [ConcreteCategory.{w} C]
99
99
100
100
-- Porting note: forget_obj_eq_coe has become a syntactic tautology.
101
101
#noalign category_theory.forget_obj_eq_coe
0 commit comments