Documentation

Mathlib.CategoryTheory.Sums.Basic

Binary disjoint unions of categories #

We define the category instance on C ⊕ D when C and D are categories.

We define:

We further define sums of functors and natural transformations, written F.sum G and α.sum β.

inl_ is the functor X ↦ inl X.

Equations
Instances For
    @[simp]
    theorem CategoryTheory.Sum.inl__map (C : Type u₁) [CategoryTheory.Category.{v₁, u₁} C] (D : Type u₁) [CategoryTheory.Category.{v₁, u₁} D] {x✝ x✝¹ : C} (f : x✝ x✝¹) :

    inr_ is the functor X ↦ inr X.

    Equations
    Instances For
      @[simp]
      theorem CategoryTheory.Sum.inr__map (C : Type u₁) [CategoryTheory.Category.{v₁, u₁} C] (D : Type u₁) [CategoryTheory.Category.{v₁, u₁} D] {x✝ x✝¹ : D} (f : x✝ x✝¹) :

      The functor exchanging two direct summand categories.

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

        swap gives an equivalence between C ⊕ D and D ⊕ C.

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

          The double swap on C ⊕ D is naturally isomorphic to the identity functor.

          Equations
          Instances For

            The sum of two functors.

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

              Similar to sum, but both functors land in the same category C

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

                The sum F.sum' G precomposed with the left inclusion functor is isomorphic to F

                Equations
                Instances For

                  The sum F.sum' G precomposed with the right inclusion functor is isomorphic to G

                  Equations
                  Instances For

                    The sum of two natural transformations.

                    Equations
                    Instances For