Documentation

Mathlib.CategoryTheory.Functor.Basic

Functors #

Defines a functor between categories, extending a Prefunctor between quivers.

Introduces, in the CategoryTheory scope, notations C ⥤ D for the type of all functors from C to D, 𝟭 for the identity functor and for functor composition.

TODO: Switch to using the arrow.

structure CategoryTheory.Functor (C : Type u₁) [CategoryTheory.Category.{v₁, u₁} C] (D : Type u₂) [CategoryTheory.Category.{v₂, u₂} D] extends Prefunctor :
Type (max v₁ v₂ u₁ u₂)

Functor C D represents a functor between categories C and D.

To apply a functor F to an object use F.obj X, and to a morphism use F.map f.

The axiom map_id expresses preservation of identities, and map_comp expresses functoriality.

See .

Instances For

    Notation for a functor between categories.

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

      𝟭 C is the identity functor on a category C.

      Equations
      • CategoryTheory.Functor.id C = { toPrefunctor := { obj := fun (X : C) => X, map := fun {X Y : C} (f : X Y) => f }, map_id := , map_comp := }
      Instances For

        Notation for the identity functor on a category.

        Equations
        Instances For
          @[simp]
          theorem CategoryTheory.Functor.id_map {C : Type u₁} [CategoryTheory.Category.{v₁, u₁} C] {X : C} {Y : C} (f : X Y) :

          F ⋙ G is the composition of a functor F and a functor G (F first, then G).

          Equations
          • CategoryTheory.Functor.comp F G = { toPrefunctor := { obj := fun (X : C) => G.obj (F.obj X), map := fun {X Y : C} (f : X Y) => G.map (F.map f) }, map_id := , map_comp := }
          Instances For

            Notation for composition of functors.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              @[simp]
              theorem CategoryTheory.Functor.map_dite {C : Type u₁} [CategoryTheory.Category.{v₁, u₁} C] {D : Type u₂} [CategoryTheory.Category.{v₂, u₂} D] (F : CategoryTheory.Functor C D) {X : C} {Y : C} {P : Prop} [Decidable P] (f : P(X Y)) (g : ¬P(X Y)) :
              F.map (if h : P then f h else g h) = if h : P then F.map (f h) else F.map (g h)