Documentation

Mathlib.CategoryTheory.Monoidal.Transport

Transport a monoidal structure along an equivalence. #

When C and D are equivalent as categories, we can transport a monoidal structure on C along the equivalence as CategoryTheory.Monoidal.transport, obtaining a monoidal structure on D.

More generally, we can transport the lawfulness of a monoidal structure along a suitable faithful functor, as CategoryTheory.Monoidal.induced. The comparison is analogous to the difference between Equiv.monoid and Function.Injective.monoid.

We then upgrade the original functor and its inverse to monoidal functors with respect to the new monoidal structure on D.

structure CategoryTheory.Monoidal.InducingFunctorData {C : Type u₁} [Category C] [MonoidalCategory C] {D : Type u₂} [Category D] [MonoidalCategoryStruct D] (F : Functor D C) :
Type (max u₂ v₁)

The data needed to induce a MonoidalCategory via the functor F; namely, pre-existing definitions of , 𝟙_, , that are preserved by F.

Instances For

    Induce the lawfulness of the monoidal structure along an faithful functor of (plain) categories, where the operations are already defined on the destination type D.

    The functor F must preserve all the data parts of the monoidal structure between the two categories.

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

      A faithful functor equipped with a InducingFunctorData structure is monoidal.

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

        Transport a monoidal structure along an equivalence of (plain) categories.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          theorem CategoryTheory.Monoidal.transportStruct_tensorHom {C : Type u₁} [Category C] [MonoidalCategory C] {D : Type u₂} [Category D] (e : Equivalence C D) {X₁✝ Y₁✝ X₂✝ Y₂✝ : D} (f : Quiver.Hom X₁✝ Y₁✝) (g : Quiver.Hom X₂✝ Y₂✝) :

          Transport a monoidal structure along an equivalence of (plain) categories.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            def CategoryTheory.Monoidal.Transported {C : Type u₁} [Category C] {D : Type u₂} [Category D] :
            Equivalence C DType u₂

            A type synonym for D, which will carry the transported monoidal structure.

            Equations
            Instances For
              @[reducible, inline]

              We upgrade the equivalence of categories e : C ≌ D to a monoidal category equivalence C ≌ Transported e.

              Equations
              Instances For

                The unit isomorphism upgrades to a monoidal isomorphism.

                The counit isomorphism upgrades to a monoidal isomorphism.