Skip to content

Commit

Permalink
fix: docstring for CategoryTheory.Limits.HasFiniteProducts (#5398)
Browse files Browse the repository at this point in the history
  • Loading branch information
kbuzzard committed Jun 23, 2023
1 parent 8eca5e6 commit ccc5499
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/CategoryTheory/Limits/Shapes/FiniteProducts.lean
Expand Up @@ -28,7 +28,7 @@ namespace CategoryTheory.Limits

variable (C : Type u) [Category.{v} C]

/-- A category has finite products if there is a chosen limit for every diagram
/-- A category has finite products if there exists a limit for every diagram
with shape `Discrete J`, where we have `[Finite J]`.
We require this condition only for `J = Fin n` in the definition, then deduce a version for any
Expand Down Expand Up @@ -62,7 +62,7 @@ theorem hasFiniteProducts_of_hasProducts [HasProducts.{w} C] : HasFiniteProducts
fun _ => hasLimitsOfShape_of_equivalence (Discrete.equivalence Equiv.ulift.{w})⟩
#align category_theory.limits.has_finite_products_of_has_products CategoryTheory.Limits.hasFiniteProducts_of_hasProducts

/-- A category has finite coproducts if there is a chosen colimit for every diagram
/-- A category has finite coproducts if there exists a colimit for every diagram
with shape `Discrete J`, where we have `[Fintype J]`.
We require this condition only for `J = Fin n` in the definition, then deduce a version for any
Expand Down

0 comments on commit ccc5499

Please sign in to comment.