Documentation

Mathlib.CategoryTheory.Distributive.Monoidal

Distributive monoidal categories #

Main definitions #

A monoidal category C with binary coproducts is left distributive if the left tensor product preserves binary coproducts. This means that, for all objects X, Y, and Z in C, the cogap map (X ⊗ Y) ⨿ (X ⊗ Z) ⟶ X ⊗ (Y ⨿ Z) can be promoted to an isomorphism. We refer to this isomorphism as the left distributivity isomorphism.

A monoidal category C with binary coproducts is right distributive if the right tensor product preserves binary coproducts. This means that, for all objects X, Y, and Z in C, the cogap map (Y ⊗ X) ⨿ (Z ⊗ X) ⟶ (Y ⨿ Z) ⊗ X can be promoted to an isomorphism. We refer to this isomorphism as the right distributivity isomorphism.

A distributive monoidal category is a monoidal category that is both left and right distributive.

Main results #

TODO #

Show that a distributive monoidal category whose unit is weakly terminal is finitary distributive.

Show that the category of pointed types with the monoidal structure given by the smash product of pointed types and the coproduct given by the wedge sum is distributive.

References #

A monoidal category with binary coproducts is left distributive if the left tensor product functor preserves binary coproducts.

Instances

    A monoidal category with binary coproducts is right distributive if the right tensor product functor preserves binary coproducts.

    Instances

      Notation for the forward direction morphism of the canonical left distributivity isomorphism

      Equations
      Instances For

        The forward direction of the left distributivity isomorphism is the cogap morphism coprod.desc (_ ◁ coprod.inl) (_ ◁ coprod.inr) : (X ⊗ Y) ⨿ (X ⊗ Z) ⟶ X ⊗ (Y ⨿ Z).

        @[simp]

        The composite of (X ◁ coprod.inl) : X ⊗ Y ⟶ X ⊗ (Y ⨿ Z) and (∂L X Y Z).inv : X ⊗ (Y ⨿ Z) ⟶ (X ⊗ Y) ⨿ (X ⊗ Z) is equal to the left coprojection coprod.inl : X ⊗ Y ⟶ (X ⊗ Y) ⨿ (X ⊗ Z).

        @[simp]

        The composite of (X ◁ coprod.inr) : X ⊗ Z ⟶ X ⊗ (Y ⨿ Z) and (∂L X Y Z).inv : X ⊗ (Y ⨿ Z) ⟶ (X ⊗ Y) ⨿ (X ⊗ Z) is equal to the right coprojection coprod.inr : X ⊗ Z ⟶ (X ⊗ Y) ⨿ (X ⊗ Z).

        Notation for the forward direction morphism of the canonical right distributivity isomorphism

        Equations
        Instances For

          The forward direction of the right distributivity isomorphism is equal to the cogap morphism coprod.desc (coprod.inl ▷ _) (coprod.inr ▷ _) : (Y ⊗ X) ⨿ (Z ⊗ X) ⟶ (Y ⨿ Z) ⊗ X.

          @[simp]

          The composite of (coprod.inl ▷ X) : Y ⊗ X ⟶ (Y ⨿ Z) ⊗ X and (∂R X Y Z).inv : (Y ⨿ Z) ⊗ X ⟶ (Y ⊗ X) ⨿ (Z ⊗ X) is equal to the left coprojection coprod.inl : Y ⊗ X ⟶ (Y ⊗ X) ⨿ (Z ⊗ X).

          @[simp]

          The composite of (coprod.inr ▷ X) : Z ⊗ X ⟶ (Y ⨿ Z) ⊗ X and (∂R X Y Z).inv : (Y ⨿ Z) ⊗ X ⟶ (Y ⊗ X) ⨿ (Z ⊗ X) is equal to the right coprojection coprod.inr : Z ⊗ X ⟶ (Y ⊗ X) ⨿ (Z ⊗ X).

          @[simp]

          In a symmetric monoidal category, the left distributivity is equal to the right distributivity up to braiding isomorphisms.

          @[simp]

          In a symmetric monoidal category, the right distributivity is equal to the left distributivity up to braiding isomorphisms.

          @[simp]

          The right distributivity isomorphism of the a left distributive symmetric monoidal category is given by (β_ (Y ⨿ Z) X).hom ≫ (∂L X Y Z).inv ≫ (coprod.map (β_ X Y).hom (β_ X Z).hom).

          The inverse of distributivity isomorphism from the closed monoidal strurcture

          The monoidal structure on the category of endofunctors is left distributive.