Documentation

Mathlib.CategoryTheory.Sums.Associator

Associator for binary disjoint union of categories. #

The associator functor ((C ⊕ D) ⊕ E) ⥤ (C ⊕ (D ⊕ E)) and its inverse form an equivalence.

def CategoryTheory.sum.associator (C : Type u) [Category.{v, u} C] (D : Type u) [Category.{v, u} D] (E : Type u) [Category.{v, u} E] :
Functor ((C D) E) (C D E)

The associator functor (C ⊕ D) ⊕ E ⥤ C ⊕ (D ⊕ E) for sums of categories.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    @[simp]
    @[simp]
    theorem CategoryTheory.sum.associator_map_inr (C : Type u) [Category.{v, u} C] (D : Type u) [Category.{v, u} D] (E : Type u) [Category.{v, u} E] {X Y : E} (f : Sum.inr X Sum.inr Y) :
    (associator C D E).map f = f

    The inverse associator functor C ⊕ (D ⊕ E) ⥤ (C ⊕ D) ⊕ E for sums of categories.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]

      The equivalence of categories expressing associativity of sums of categories.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For