Comonadic adjunctions🔗
An adjunction
between functors
and
is comonadic if the induced comparison functor
(where the right-hand side is the category of Coalgebras
of the comonad of the
adjunction) is an equivalence of categories. This dualises the
theory of monadic adjunctions.
module Cat.Functor.Adjoint.Comonadic {o₁ h₁ o₂ h₂ : _} {C : Precategory o₁ h₁} {D : Precategory o₂ h₂} {L : Functor C D} {R : Functor D C} (L⊣R : L ⊣ R) where
private module C = Cat.Reasoning C module D = Cat.Reasoning D module L = Cat.Functor.Reasoning L module R = Cat.Functor.Reasoning R module adj = _⊣_ L⊣R L∘R : Comonad-on _ L∘R = Adjunction→Comonad L⊣R open Comonad-on L∘R _ = Coalgebra
The composition of L.₁
with
the adjunction unit
natural
transformation gives L
a Coalgebra
structure, thus
extending L
to a functor
Comparison-CoEM : Functor C (Coalgebras L∘R) Comparison-CoEM .F₀ x = L.₀ x , alg where alg : Coalgebra-on L∘R (L.₀ x) alg .Coalgebra-on.ρ = L.₁ (adj.unit.η _) alg .Coalgebra-on.ρ-counit = adj.zig alg .Coalgebra-on.ρ-comult = L.weave (adj.unit.is-natural _ _ _)
Construction of the functorial action of Comparison-CoEM
Comparison-CoEM .F₁ x .fst = L.₁ x Comparison-CoEM .F₁ x .snd = L.weave (sym (adj.unit.is-natural _ _ _)) Comparison-CoEM .F-id = ext L.F-id Comparison-CoEM .F-∘ f g = ext (L.F-∘ _ _)
By construction, the composition of the comparison functor with the forgetful functor is equal to
Forget∘Comparison≡L : πᶠ (Coalgebras-over L∘R) F∘ Comparison-CoEM ≡ L Forget∘Comparison≡L = Functor-path (λ _ → refl) (λ _ → refl)
An adjunction is comonadic if Comparison-CoEM
is an equivalence of categories, thus
exhibiting
as the category of
is-comonadic : Type _ is-comonadic = is-equivalence Comparison-CoEM
We also say that the left adjoint is a comonadic functor.
Comonadic functors create colimits🔗
By the description of colimits in
categories of coalgebras, the forgetful functor πᶠ
creates colimits.
Furthermore, if the adjunction
is comonadic, then Comparison-CoEM
is an
equivalence of categories, so it also creates colimits. Since this
property is closed under composition, comonadic functors creates
colimits.
comonadic→creates-colimits : ∀ {oj ℓj} {J : Precategory oj ℓj} → creates-colimits-of J L comonadic→creates-colimits = subst (creates-colimits-of _) Forget∘Comparison≡L $ F∘-creates-colimits (equivalence→creates-colimits comonadic) (Forget-CoEM-creates-colimits L∘R)