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

Commit 3947876

Browse files
committed
chore(category_theory/limits/preserves): fix typo (#18906)
1 parent 8130e51 commit 3947876

File tree

2 files changed

+3
-3
lines changed

2 files changed

+3
-3
lines changed

src/category_theory/functor/flat.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -355,7 +355,7 @@ begin
355355
haveI : preserves_finite_limits F :=
356356
begin
357357
apply preserves_finite_limits_of_preserves_finite_limits_of_size.{u₁},
358-
intros, resetI, apply preserves_limit_of_Lan_presesrves_limit
358+
intros, resetI, apply preserves_limit_of_Lan_preserves_limit
359359
end,
360360
apply flat_of_preserves_finite_limits
361361
end
@@ -371,7 +371,7 @@ def preserves_finite_limits_iff_Lan_preserves_finite_limits (F : C ⥤ D) :
371371
inv_fun := λ _,
372372
begin
373373
apply preserves_finite_limits_of_preserves_finite_limits_of_size.{u₁},
374-
intros, resetI, apply preserves_limit_of_Lan_presesrves_limit
374+
intros, resetI, apply preserves_limit_of_Lan_preserves_limit
375375
end,
376376
left_inv := λ x,
377377
begin

src/category_theory/limits/preserves/functor_category.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -99,7 +99,7 @@ instance whiskering_right_preserves_limits {C : Type u} [category C]
9999

100100
/-- If `Lan F.op : (Cᵒᵖ ⥤ Type*) ⥤ (Dᵒᵖ ⥤ Type*)` preserves limits of shape `J`, so will `F`. -/
101101
noncomputable
102-
def preserves_limit_of_Lan_presesrves_limit {C D : Type u} [small_category C] [small_category D]
102+
def preserves_limit_of_Lan_preserves_limit {C D : Type u} [small_category C] [small_category D]
103103
(F : C ⥤ D) (J : Type u) [small_category J]
104104
[preserves_limits_of_shape J (Lan F.op : _ ⥤ (Dᵒᵖ ⥤ Type u))] :
105105
preserves_limits_of_shape J F :=

0 commit comments

Comments
 (0)