Skip to content

Commit

Permalink
chore(category_theory/limits/preserves): fix typo (#18906)
Browse files Browse the repository at this point in the history
  • Loading branch information
kbuzzard committed May 1, 2023
1 parent 8130e51 commit 3947876
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 3 deletions.
4 changes: 2 additions & 2 deletions src/category_theory/functor/flat.lean
Expand Up @@ -355,7 +355,7 @@ begin
haveI : preserves_finite_limits F :=
begin
apply preserves_finite_limits_of_preserves_finite_limits_of_size.{u₁},
intros, resetI, apply preserves_limit_of_Lan_presesrves_limit
intros, resetI, apply preserves_limit_of_Lan_preserves_limit
end,
apply flat_of_preserves_finite_limits
end
Expand All @@ -371,7 +371,7 @@ def preserves_finite_limits_iff_Lan_preserves_finite_limits (F : C ⥤ D) :
inv_fun := λ _,
begin
apply preserves_finite_limits_of_preserves_finite_limits_of_size.{u₁},
intros, resetI, apply preserves_limit_of_Lan_presesrves_limit
intros, resetI, apply preserves_limit_of_Lan_preserves_limit
end,
left_inv := λ x,
begin
Expand Down
2 changes: 1 addition & 1 deletion src/category_theory/limits/preserves/functor_category.lean
Expand Up @@ -99,7 +99,7 @@ instance whiskering_right_preserves_limits {C : Type u} [category C]

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

0 comments on commit 3947876

Please sign in to comment.