Documentation

Mathlib.CategoryTheory.Extensive

Extensive categories #

Main definitions #

Main Results #

TODO #

Show that the following are finitary extensive:

References #

A category has pullback of inclusions if it has all pullbacks along coproduct injections.

Instances

    A functor preserves pullback of inclusions if it preserves all pullbacks along coproduct injections.

    Instances

      A category is (finitary) pre-extensive if it has finite coproducts, and binary coproducts are universal.

      Instances

        A category is (finitary) extensive if it has finite coproducts, and binary coproducts are van Kampen.

        Instances
          Equations
          • One or more equations did not get rendered due to their size.
          Equations
          • One or more equations did not get rendered due to their size.
          Equations
          • =
          theorem CategoryTheory.FinitaryPreExtensive.sigma_desc_iso {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.FinitaryPreExtensive C] {α : Type} [Finite α] {X : C} {Z : αC} (π : (a : α) → Z a X) {Y : C} (f : Y X) (hπ : CategoryTheory.IsIso (CategoryTheory.Limits.Sigma.desc π)) :
          CategoryTheory.IsIso (CategoryTheory.Limits.Sigma.desc fun (x : α) => CategoryTheory.Limits.pullback.fst)