Modifications between transformations of oplax functors #
In this file we define modifications of oplax and strong transformations of oplax functors.
A modification Γ between oplax transformations η and θ (of oplax functors) consists of a
family of 2-morphisms Γ.app a : η.app a ⟶ θ.app a, which for all 1-morphisms f : a ⟶ b
satisfies the equation (F.map f ◁ app b) ≫ θ.naturality f = η.naturality f ≫ (app a ▷ G.map f).
Modifications between strong transformations are defined similarly.
Main definitions #
Given two oplax functors F and G, we define:
OplaxTrans.Modification η θ: modifications between oplax transformationsηandθbetweenFandG.OplaxTrans.homCategory F G: the category structure on the oplax transformations betweenFandG, where composition is given by vertical composition. Note that this a scoped instance in theOplax.OplaxTransnamespace, so you need to runopen scoped Oplax.OplaxTransto access it.StrongTrans.Modification η θ: modifications between strong transformationsηandθbetweenFandG.StrongTrans.homCategory F G: the category structure on the strong transformations betweenFandG, where composition is given by vertical composition. Note that this a scoped instance in theOplax.StrongTransnamespace, so you need to runopen scoped Oplax.StrongTransto access it.
A modification Γ between oplax natural transformations η and θ consists of a family of
2-morphisms Γ.app a : η.app a ⟶ θ.app a, which satisfies the equation
(F.map f ◁ app b) ≫ θ.naturality f = η.naturality f ≫ (app a ▷ G.map f)
for each 1-morphism f : a ⟶ b.
The underlying family of 2-morphisms.
- naturality {a b : B} (f : a ⟶ b) : CategoryStruct.comp (Bicategory.whiskerLeft (F.map f) (self.app b)) (θ.naturality f) = CategoryStruct.comp (η.naturality f) (Bicategory.whiskerRight (self.app a) (G.map f))
The naturality condition.
Instances For
The identity modification.
Equations
- CategoryTheory.Oplax.OplaxTrans.Modification.id η = { app := fun (a : B) => CategoryTheory.CategoryStruct.id (η.app a), naturality := ⋯ }
Instances For
Vertical composition of modifications.
Equations
Instances For
Category structure on the oplax natural transformations between OplaxFunctors.
Note that this a scoped instance in the Oplax.OplaxTrans namespace.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Version of Modification.id_app using category notation
Version of Modification.comp_app using category notation
Construct a modification isomorphism between oplax natural transformations by giving object level isomorphisms, and checking naturality only in the forward direction.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Alias of CategoryTheory.Oplax.OplaxTrans.isoMk.
Construct a modification isomorphism between oplax natural transformations by giving object level isomorphisms, and checking naturality only in the forward direction.
Equations
Instances For
A modification Γ between strong natural transformations η and θ (between oplax functors)
consists of a family of 2-morphisms Γ.app a : η.app a ⟶ θ.app a, which satisfies the equation
(F.map f ◁ app b) ≫ (θ.naturality f).hom = (η.naturality f).hom ≫ (app a ▷ G.map f)
for each 1-morphism f : a ⟶ b.
The underlying family of 2-morphisms.
- naturality {a b : B} (f : a ⟶ b) : CategoryStruct.comp (Bicategory.whiskerLeft (F.map f) (self.app b)) (θ.naturality f).hom = CategoryStruct.comp (η.naturality f).hom (Bicategory.whiskerRight (self.app a) (G.map f))
The naturality condition.
Instances For
The modification between the underlying strong transformations of oplax functors
Instances For
The modification between strong transformations of oplax functors associated to a modification between the underlying oplax transformations.
Equations
- CategoryTheory.Oplax.StrongTrans.Modification.mkOfOplax Γ = { app := fun (a : B) => Γ.app a, naturality := ⋯ }
Instances For
Modifications between strong transformations of oplax functors are equivalent to modifications between the underlying oplax transformations.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The identity modification.
Equations
- CategoryTheory.Oplax.StrongTrans.Modification.id η = { app := fun (a : B) => CategoryTheory.CategoryStruct.id (η.app a), naturality := ⋯ }
Instances For
Vertical composition of modifications.
Equations
Instances For
Category structure on the strong natural transformations between oplax functors.
Note that this a scoped instance in the Oplax.StrongTrans namespace.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Construct a modification isomorphism between strong natural transformations (of oplax functors) by giving object level isomorphisms, and checking naturality only in the forward direction.
Equations
- One or more equations did not get rendered due to their size.