Documentation

Mathlib.CategoryTheory.Category.Quiv

The category of quivers #

The category of (bundled) quivers, and the free/forgetful adjunction between Cat and Quiv.

def CategoryTheory.Quiv :
Type (max (u + 1) u (v + 1))

Category of quivers.

Equations
Instances For

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

    Equations
    Instances For
      @[simp]
      theorem CategoryTheory.Quiv.forget_map :
      ∀ {X Y : CategoryTheory.Cat} (F : X Y), CategoryTheory.Quiv.forget.map F = F.toPrefunctor

      The forgetful functor from categories to quivers.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[simp]
        theorem CategoryTheory.Cat.free_map_map :
        ∀ {X Y : CategoryTheory.Quiv} (F : X Y) {X_1 Y_1 : ((fun (V : CategoryTheory.Quiv) => CategoryTheory.Cat.of (CategoryTheory.Paths V)) X)} (f : X_1 Y_1), (CategoryTheory.Cat.free.map F).map f = Prefunctor.mapPath F f
        @[simp]
        theorem CategoryTheory.Cat.free_map_obj :
        ∀ {X Y : CategoryTheory.Quiv} (F : X Y) (X_1 : ((fun (V : CategoryTheory.Quiv) => CategoryTheory.Cat.of (CategoryTheory.Paths V)) X)), (CategoryTheory.Cat.free.map F).obj X_1 = F.obj X_1

        The functor sending each quiver to its path category.

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

          Any prefunctor into a category lifts to a functor from the path category.

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

            The adjunction between forming the free category on a quiver, and forgetting a category to a quiver.

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