@@ -27,15 +27,15 @@ namespace CategoryTheory
27
27
28
28
open Category Limits
29
29
30
- universe w' w v u₁ u₂ u₃
30
+ universe w' w v₁ v₂ v₃ u₁ u₂ u₃
31
31
32
32
variable {J : Type w} [Category.{w'} J]
33
33
34
- variable {A : Type u₁} [Category.{v} A]
34
+ variable {A : Type u₁} [Category.{v₁ } A]
35
35
36
- variable {B : Type u₂} [Category.{v} B]
36
+ variable {B : Type u₂} [Category.{v₂ } B]
37
37
38
- variable {T : Type u₃} [Category.{v} T]
38
+ variable {T : Type u₃} [Category.{v₃ } T]
39
39
40
40
namespace Comma
41
41
@@ -153,9 +153,10 @@ instance hasLimitsOfShape [HasLimitsOfShape J A] [HasLimitsOfShape J B]
153
153
[PreservesLimitsOfShape J R] : HasLimitsOfShape J (Comma L R) where
154
154
#align category_theory.comma.has_limits_of_shape CategoryTheory.Comma.hasLimitsOfShape
155
155
156
- instance hasLimits [HasLimits A] [HasLimits B] [PreservesLimits R] : HasLimits (Comma L R) :=
156
+ instance hasLimitsOfSize [HasLimitsOfSize.{w, w'} A] [HasLimitsOfSize.{w, w'} B]
157
+ [PreservesLimitsOfSize.{w, w'} R] : HasLimitsOfSize.{w, w'} (Comma L R) :=
157
158
⟨fun _ _ => inferInstance⟩
158
- #align category_theory.comma.has_limits CategoryTheory.Comma.hasLimits
159
+ #align category_theory.comma.has_limits CategoryTheory.Comma.hasLimitsOfSize
159
160
160
161
instance hasColimit (F : J ⥤ Comma L R) [HasColimit (F ⋙ fst L R)] [HasColimit (F ⋙ snd L R)]
161
162
[PreservesColimit (F ⋙ fst L R) L] : HasColimit F :=
@@ -166,10 +167,10 @@ instance hasColimitsOfShape [HasColimitsOfShape J A] [HasColimitsOfShape J B]
166
167
[PreservesColimitsOfShape J L] : HasColimitsOfShape J (Comma L R) where
167
168
#align category_theory.comma.has_colimits_of_shape CategoryTheory.Comma.hasColimitsOfShape
168
169
169
- instance hasColimits [HasColimits A] [HasColimits B] [PreservesColimits L] :
170
- HasColimits (Comma L R) :=
170
+ instance hasColimitsOfSize [HasColimitsOfSize.{w, w'} A] [HasColimitsOfSize.{w, w'} B]
171
+ [PreservesColimitsOfSize.{w, w'} L] : HasColimitsOfSize.{w, w'} (Comma L R) :=
171
172
⟨fun _ _ => inferInstance⟩
172
- #align category_theory.comma.has_colimits CategoryTheory.Comma.hasColimits
173
+ #align category_theory.comma.has_colimits CategoryTheory.Comma.hasColimitsOfSize
173
174
174
175
end Comma
175
176
@@ -220,9 +221,10 @@ instance hasLimitsOfShape [HasLimitsOfShape J A] [PreservesLimitsOfShape J G] :
220
221
HasLimitsOfShape J (StructuredArrow X G) where
221
222
#align category_theory.structured_arrow.has_limits_of_shape CategoryTheory.StructuredArrow.hasLimitsOfShape
222
223
223
- instance hasLimits [HasLimits A] [PreservesLimits G] : HasLimits (StructuredArrow X G) :=
224
+ instance hasLimitsOfSize [HasLimitsOfSize.{w, w'} A] [PreservesLimitsOfSize.{w, w'} G] :
225
+ HasLimitsOfSize.{w, w'} (StructuredArrow X G) :=
224
226
⟨fun J hJ => by infer_instance⟩
225
- #align category_theory.structured_arrow.has_limits CategoryTheory.StructuredArrow.hasLimits
227
+ #align category_theory.structured_arrow.has_limits CategoryTheory.StructuredArrow.hasLimitsOfSize
226
228
227
229
noncomputable instance createsLimit [i : PreservesLimit (F ⋙ proj X G) G] :
228
230
CreatesLimit F (proj X G) :=
@@ -237,8 +239,9 @@ noncomputable instance createsLimitsOfShape [PreservesLimitsOfShape J G] :
237
239
CreatesLimitsOfShape J (proj X G) where
238
240
#align category_theory.structured_arrow.creates_limits_of_shape CategoryTheory.StructuredArrow.createsLimitsOfShape
239
241
240
- noncomputable instance createsLimits [PreservesLimits G] : CreatesLimits (proj X G : _) where
241
- #align category_theory.structured_arrow.creates_limits CategoryTheory.StructuredArrow.createsLimits
242
+ noncomputable instance createsLimitsOfSize [PreservesLimitsOfSize.{w, w'} G] :
243
+ CreatesLimitsOfSize.{w, w'} (proj X G : _) where
244
+ #align category_theory.structured_arrow.creates_limits CategoryTheory.StructuredArrow.createsLimitsOfSize
242
245
243
246
instance mono_right_of_mono [HasPullbacks A] [PreservesLimitsOfShape WalkingCospan G]
244
247
{Y Z : StructuredArrow X G} (f : Y ⟶ Z) [Mono f] : Mono f.right :=
@@ -267,9 +270,10 @@ instance hasColimitsOfShape [HasColimitsOfShape J A] [PreservesColimitsOfShape J
267
270
HasColimitsOfShape J (CostructuredArrow G X) where
268
271
#align category_theory.costructured_arrow.has_colimits_of_shape CategoryTheory.CostructuredArrow.hasColimitsOfShape
269
272
270
- instance hasColimits [HasColimits A] [PreservesColimits G] : HasColimits (CostructuredArrow G X) :=
273
+ instance hasColimitsOfSize [HasColimitsOfSize.{w, w'} A] [PreservesColimitsOfSize.{w, w'} G] :
274
+ HasColimitsOfSize.{w, w'} (CostructuredArrow G X) :=
271
275
⟨fun _ _ => inferInstance⟩
272
- #align category_theory.costructured_arrow.has_colimits CategoryTheory.CostructuredArrow.hasColimits
276
+ #align category_theory.costructured_arrow.has_colimits CategoryTheory.CostructuredArrow.hasColimitsOfSize
273
277
274
278
noncomputable instance createsColimit [i : PreservesColimit (F ⋙ proj G X) G] :
275
279
CreatesColimit F (proj G X) :=
@@ -284,8 +288,9 @@ noncomputable instance createsColimitsOfShape [PreservesColimitsOfShape J G] :
284
288
CreatesColimitsOfShape J (proj G X) where
285
289
#align category_theory.costructured_arrow.creates_colimits_of_shape CategoryTheory.CostructuredArrow.createsColimitsOfShape
286
290
287
- noncomputable instance createsColimits [PreservesColimits G] : CreatesColimits (proj G X : _) where
288
- #align category_theory.costructured_arrow.creates_colimits CategoryTheory.CostructuredArrow.createsColimits
291
+ noncomputable instance createsColimitsOfSize [PreservesColimitsOfSize.{w, w'} G] :
292
+ CreatesColimitsOfSize.{w, w'} (proj G X : _) where
293
+ #align category_theory.costructured_arrow.creates_colimits CategoryTheory.CostructuredArrow.createsColimitsOfSize
289
294
290
295
instance epi_left_of_epi [HasPushouts A] [PreservesColimitsOfShape WalkingSpan G]
291
296
{Y Z : CostructuredArrow G X} (f : Y ⟶ Z) [Epi f] : Epi f.left :=
0 commit comments