Documentation

Mathlib.CategoryTheory.Monoidal.Action.Opposites

Actions from the monoidal opposite of a category. #

In this file, given a monoidal category C and a category D, we construct a left C-action on D out of the data of a right Cᴹᵒᵖ-action on D. We also construct a right C-action on Dfrom the data of a left Cᴹᵒᵖ-action on D. Conversely, given left/right C-actions on D, we construct aCᴹᵒᵖ actions with the conjugate variance.

These constructions are not made instances in order to avoid instance loops, you should bring them as local instances if you intend to use them.

Define a left action of C on D from a right action of Cᴹᵒᵖ on D via the formula c ⊙ₗ d := d ⊙ᵣ (mop c).

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

    Define a left action of Cᴹᵒᵖ on D from a right action of C on D via the formula mop c ⊙ₗ d = d ⊙ᵣ c.

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

      Define a right action of C on D from a left action of Cᴹᵒᵖ on D via the formula d ⊙ᵣ c := (mop c) ⊙ₗ d.

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

        Define a right action of Cᴹᵒᵖ on D from a left action of C on D via the formula d ⊙ᵣ mop c = c ⊙ₗ d.

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