Dinatural transformations #
Dinatural transformations are special kinds of transformations between
functors F G : Cᵒᵖ ⥤ C ⥤ D
which depend both covariantly and contravariantly
on the same category (also known as difunctors).
A dinatural transformation is a family of morphisms given only on the diagonal of the two functors, and is such that a certain naturality hexagon commutes. Note that dinatural transformations cannot be composed with each other (since the outer hexagon does not commute in general), but can still be "pre/post-composed" with ordinary natural transformations.
References #
Dinatural transformations between two difunctors.
The component of a natural transformation.
- dinaturality {X Y : C} (f : X ⟶ Y) : CategoryStruct.comp ((F.map f.op).app X) (CategoryStruct.comp (self.app X) ((G.obj (Opposite.op X)).map f)) = CategoryStruct.comp ((F.obj (Opposite.op Y)).map f) (CategoryStruct.comp (self.app Y) ((G.map f.op).app Y))
The commutativity square for a given morphism.
Instances For
Notation for dinatural transformations.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Post-composition with a natural transformation.
Equations
- δ.compNatTrans α = { app := fun (X : C) => CategoryTheory.CategoryStruct.comp (δ.app X) ((α.app (Opposite.op X)).app X), dinaturality := ⋯ }
Instances For
Pre-composition with a natural transformation.
Equations
- δ.precompNatTrans α = { app := fun (X : C) => CategoryTheory.CategoryStruct.comp ((α.app (Opposite.op X)).app X) (δ.app X), dinaturality := ⋯ }