Natural transformations #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Defines natural transformations between functors.
A natural transformation α : nat_trans 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 nat_trans.naturality
a simp lemma, with the preferred simp normal form
pushing components of natural transformations to the left.
See also category_theory.functor_category
, where we provide the category structure on
functors and natural transformations.
Introduces notations
τ.app X
for the components of natural transformations,F ⟶ G
for the type of natural transformations between functorsF
andG
(this and the next requirecategory_theory.functor_category
),σ ≫ τ
for vertical compositions, andσ ◫ τ
for horizontal compositions.
- app : Π (X : C), F.obj X ⟶ G.obj X
- naturality' : (∀ ⦃X Y : C⦄ (f : X ⟶ Y), F.map f ≫ self.app Y = self.app X ≫ G.map f) . "obviously"
nat_trans 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_lemma
.
Instances for category_theory.nat_trans
- category_theory.nat_trans.has_sizeof_inst
- category_theory.nat_trans.inhabited
nat_trans.id F
is the identity natural transformation on a functor F
.
Equations
- category_theory.nat_trans.id F = {app := λ (X : C), 𝟙 (F.obj X), naturality' := _}
Equations
vcomp α β
is the vertical compositions of natural transformations.