Comonads in a bicategory #
We define comonads in a bicategory B
as comonoid objects in an endomorphism monoidal category.
We show that this is equivalent to oplax functors from the trivial bicategory to B
. From this,
we show that comonads in B
form a bicategory.
TODO #
We can also define monads in a bicategory. This is not yet done as we don't have the bicategory structure on the set of lax functors at this point, which is needed to show that monads form a bicategory.
A comonad in a bicategory B
is a 1-morphism t : a ⟶ a
together with 2-morphisms
Δ : t ⟶ t ≫ t
and ε : t ⟶ 𝟙 a
satisfying the comonad laws.
Equations
Instances For
The counit 2-morphism of the comonad.
Instances For
The comultiplication 2-morphism of the comonad.
Instances For
The counit 2-morphism of the comonad.
Equations
- CategoryTheory.Bicategory.termε = Lean.ParserDescr.node `CategoryTheory.Bicategory.termε 1024 (Lean.ParserDescr.symbol "ε")
Instances For
The counit 2-morphism of the comonad.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The comultiplication 2-morphism of the comonad.
Equations
- CategoryTheory.Bicategory.termΔ = Lean.ParserDescr.node `CategoryTheory.Bicategory.termΔ 1024 (Lean.ParserDescr.symbol "Δ")
Instances For
The comultiplication 2-morphism of the comonad.
Equations
- One or more equations did not get rendered due to their size.
Instances For
An oplax functor from the trivial bicategory to B
defines a comonad in B
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A comonad in B
defines an oplax functor from the trivial bicategory to B
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The bicategory of comonads in B
.
Equations
Instances For
The bicategory of comonads in B
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The oplax functor from the trivial bicategory to B
associated with the comonad.
Instances For
The object in B
associated with the comonad.
Instances For
The morphism in B
associated with the comonad.
Equations
- m.hom = m.toOplax.map (CategoryTheory.CategoryStruct.id { as := { as := PUnit.unit } })
Instances For
Construct a comonad as an object in ComonadBicat B
.