Documentation

Mathlib.Tactic.CategoryTheory.Monoidal.Datatypes

Expressions for monoidal categories #

This file converts lean expressions representing morphisms in monoidal categories into Mor₂Iso or Mor terms. The converted expressions are used in the coherence tactics and the string diagram widgets.

The domain of a morphism.

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

    The codomain of a morphism.

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

      The domain of an isomorphism.

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

        The codomain of an isomorphism.

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

          The context for evaluating expressions.

          Instances For

            Populate a context object for evaluating e.

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

              The monad for the normalization of 2-morphisms.

              Equations
              Instances For

                Throw an error if the monoidal category instance is not found.

                Equations
                Instances For
                  Equations
                  • One or more equations did not get rendered due to their size.
                  theorem Mathlib.Tactic.Monoidal.structuralIsoOfExpr_comp {C : Type u} [CategoryTheory.Category.{v, u} C] {f g h : C} (η : f g) (η' : f g) (ih_η : η'.hom = η) (θ : g h) (θ' : g h) (ih_θ : θ'.hom = θ) :
                  theorem Mathlib.Tactic.Monoidal.StructuralOfExpr_monoidalComp {C : Type u} [CategoryTheory.Category.{v, u} C] {f g h i : C} [CategoryTheory.MonoidalCoherence g h] (η : f g) (η' : f g) (ih_η : η'.hom = η) (θ : h i) (θ' : h i) (ih_θ : θ'.hom = θ) :
                  theorem Mathlib.Tactic.Monoidal.structuralIsoOfExpr_horizontalComp {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.MonoidalCategory C] {f₁ g₁ f₂ g₂ : C} (η : f₁ g₁) (η' : f₁ g₁) (ih_η : η'.hom = η) (θ : f₂ g₂) (θ' : f₂ g₂) (ih_θ : θ'.hom = θ) :
                  Equations
                  • One or more equations did not get rendered due to their size.
                  Equations
                  • One or more equations did not get rendered due to their size.

                  Check that e is definitionally equal to 𝟙_ C.

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

                    Return (f, g) if e is definitionally equal to f ⊗ g.

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

                      Construct a Mor₁ expression from a Lean expression.

                      Construct a Mor₂Iso term from a Lean expression.

                      Construct a Mor₂ term from a Lean expression.