Documentation

Mathlib.CategoryTheory.NatTrans

Natural transformations #

Defines natural transformations between functors.

A natural transformation α : NatTrans F G consists of morphisms α.app X : F.obj X ⟶ G.obj X, and the naturality squares α.naturality f : F.map f ≫ α.app Y = α.app X ≫ G.map f, where f : X ⟶ Y.

Note that we make NatTrans.naturality a simp lemma, with the preferred simp normal form pushing components of natural transformations to the left.

See also CategoryTheory.FunctorCat, where we provide the category structure on functors and natural transformations.

Introduces notations

theorem CategoryTheory.NatTrans.ext {C : Type u₁} :
∀ {inst : CategoryTheory.Category.{v₁, u₁} C} {D : Type u₂} {inst_1 : CategoryTheory.Category.{v₂, u₂} D} {F G : CategoryTheory.Functor C D} (x y : F.NatTrans G), x.app = y.appx = y
theorem CategoryTheory.NatTrans.ext_iff {C : Type u₁} :
∀ {inst : CategoryTheory.Category.{v₁, u₁} C} {D : Type u₂} {inst_1 : CategoryTheory.Category.{v₂, u₂} D} {F G : CategoryTheory.Functor C D} (x y : F.NatTrans G), x = y x.app = y.app

NatTrans F G represents a natural transformation between functors F and G.

The field app provides the components of the natural transformation.

Naturality is expressed by α.naturality.

Instances For
    @[simp]
    theorem CategoryTheory.NatTrans.naturality_assoc {C : Type u₁} [CategoryTheory.Category.{v₁, u₁} C] {D : Type u₂} [CategoryTheory.Category.{v₂, u₂} D] {F : CategoryTheory.Functor C D} {G : CategoryTheory.Functor C D} (self : F.NatTrans G) ⦃X : C ⦃Y : C (f : X Y) {Z : D} (h : G.obj Y Z) :
    theorem CategoryTheory.congr_app {C : Type u₁} [CategoryTheory.Category.{v₁, u₁} C] {D : Type u₂} [CategoryTheory.Category.{v₂, u₂} D] {F : CategoryTheory.Functor C D} {G : CategoryTheory.Functor C D} {α : F.NatTrans G} {β : F.NatTrans G} (h : α = β) (X : C) :
    α.app X = β.app X

    NatTrans.id F is the identity natural transformation on a functor F.

    Equations
    Instances For
      def CategoryTheory.NatTrans.vcomp {C : Type u₁} [CategoryTheory.Category.{v₁, u₁} C] {D : Type u₂} [CategoryTheory.Category.{v₂, u₂} D] {F : CategoryTheory.Functor C D} {G : CategoryTheory.Functor C D} {H : CategoryTheory.Functor C D} (α : F.NatTrans G) (β : G.NatTrans H) :
      F.NatTrans H

      vcomp α β is the vertical compositions of natural transformations.

      Equations
      Instances For