Documentation

Mathlib.CategoryTheory.Limits.FintypeCat

(Co)limits in the category of finite types #

We show that finite (co)limits exist in FintypeCat and that they are preserved by the natural inclusion FintypeCat.incl.

Any functor from a finite category to Types that only involves finite objects, has a finite limit.

Equations
Equations
  • CategoryTheory.Limits.FintypeCat.instCreatesLimitsOfShapeFintypeCatForgetOfFinCategory = CategoryTheory.Limits.FintypeCat.inclusionCreatesFiniteLimits
Equations
  • One or more equations did not get rendered due to their size.
noncomputable def CategoryTheory.Limits.FintypeCat.productEquiv {ι : Type u_1} [Finite ι] (X : ιFintypeCat) :
(∏ᶜ X) ((i : ι) → (X i))

The categorical product of a finite family in FintypeCat is equivalent to the product as types.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    instance CategoryTheory.Limits.FintypeCat.nonempty_pi_of_nonempty {ι : Type u_1} [Finite ι] (X : ιFintypeCat) [∀ (i : ι), Nonempty (X i)] :
    Equations
    • =
    Equations
    • CategoryTheory.Limits.FintypeCat.instCreatesColimitsOfShapeFintypeCatForgetOfFinCategory = CategoryTheory.Limits.FintypeCat.inclusionCreatesFiniteColimits
    Equations
    • One or more equations did not get rendered due to their size.