Documentation

Mathlib.CategoryTheory.Enriched.EnrichedCat

The bicategory of V-enriched categories #

We define the bicategory EnrichedCat V of (bundled) V-enriched categories for a fixed monoidal category V.

Future work #

def CategoryTheory.EnrichedCat (V : Type v) [Category.{w, v} V] [MonoidalCategory V] :
Type (max (u + 1) (max u v) w)

Category of V-enriched categories for a monoidal category V.

Equations
Instances For

    Construct a bundled EnrichedCat from the underlying type and the typeclass.

    Equations
    Instances For

      Whisker a V-enriched natural transformation on the left.

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

        Whisker a V-enriched natural transformation on the right.

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

          Composing the V-enriched identity functor with any functor is isomorphic to that functor.

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

            Composing any V-enriched functor with the identity functor is isomorphic to the former functor.

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

              Composition of V-enriched functors is associative up to isomorphism.

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

                The bicategory structure on EnrichedCat V for a monoidal category V.

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