The continuation monad
Content created by Egbert Rijke and Fredrik Bakke.
Created on 2024-11-05.
Last modified on 2024-11-05.
module foundation.continuations where
Imports
open import foundation.action-on-identifications-functions open import foundation.dependent-pair-types open import foundation.empty-types open import foundation.equality-cartesian-product-types open import foundation.evaluation-functions open import foundation.function-extensionality open import foundation.logical-equivalences open import foundation.type-arithmetic-cartesian-product-types open import foundation.type-arithmetic-dependent-function-types open import foundation.type-arithmetic-empty-type open import foundation.type-arithmetic-unit-type open import foundation.unit-type open import foundation.universal-property-cartesian-product-types open import foundation.universal-property-empty-type open import foundation.universal-property-equivalences open import foundation.universe-levels open import foundation-core.cartesian-product-types open import foundation-core.equivalences open import foundation-core.function-types open import foundation-core.homotopies open import foundation-core.identity-types open import foundation-core.propositions open import foundation-core.retractions open import foundation-core.sections open import foundation-core.transport-along-identifications open import orthogonal-factorization-systems.extensions-of-maps open import orthogonal-factorization-systems.local-types open import orthogonal-factorization-systems.modal-operators open import orthogonal-factorization-systems.uniquely-eliminating-modalities
Idea
Given a type R
, the
continuation monad¶
on R
is the functorial construction defined on types by
A ↦ ((A → R) → R).
Definitions
The operator of the continuation monad
continuation : {l1 l2 : Level} (R : UU l1) (A : UU l2) → UU (l1 ⊔ l2) continuation R A = (A → R) → R
The functorial action of the continuation monad on maps
map-continuation : {l1 l2 l3 : Level} {R : UU l1} {A : UU l2} {B : UU l3} → (A → B) → continuation R A → continuation R B map-continuation f c g = c (g ∘ f)
The unit of the continuation monad
unit-continuation : {l1 l2 : Level} {R : UU l1} {A : UU l2} → A → continuation R A unit-continuation = ev
Maps into continuation R A
extend along the unit
Every f
as in the following diagram
extends along the unit
of its domain
f
A -------> continuation R B
| ∧
η_A | ⋰
∨ ⋰
continuation R A.
module _ {l1 l2 l3 : Level} {R : UU l1} {A : UU l2} {B : UU l3} where extend-continuation : (A → continuation R B) → (continuation R A → continuation R B) extend-continuation f c g = c (λ a → f a g) is-extension-extend-continuation : (f : A → continuation R B) → is-extension unit-continuation f (extend-continuation f) is-extension-extend-continuation f = refl-htpy extension-continuation : (f : A → continuation R B) → extension unit-continuation f extension-continuation f = ( extend-continuation f , is-extension-extend-continuation f)
The monoidal multiplication operation of the continuation monad
mul-continuation : {l1 l2 : Level} {R : UU l1} {A : UU l2} → continuation R (continuation R A) → continuation R A mul-continuation f c = f (ev c)
Properties
The right unit law for the continuation monad
module _ {l1 l2 : Level} {R : UU l1} {A : UU l2} where right-unit-law-mul-continuation : mul-continuation {R = R} ∘ unit-continuation {R = R} {continuation R A} ~ id right-unit-law-mul-continuation = refl-htpy
The continuation monad on propositions gives propositions
is-prop-continuation : {l1 l2 : Level} {R : UU l1} {A : UU l2} → is-prop R → is-prop (continuation R A) is-prop-continuation = is-prop-function-type is-prop-continuation-Prop : {l1 l2 : Level} (R : Prop l1) {A : UU l2} → is-prop (continuation (type-Prop R) A) is-prop-continuation-Prop R = is-prop-continuation (is-prop-type-Prop R) continuation-Prop : {l1 l2 : Level} (R : Prop l1) (A : UU l2) → Prop (l1 ⊔ l2) continuation-Prop R A = ( continuation (type-Prop R) A , is-prop-continuation (is-prop-type-Prop R))
Computing continuation R
on the unit type
We have the equivalence
continuation R unit ≃ (R → R).
module _ {l1 : Level} {R : UU l1} where compute-unit-continuation : continuation R unit ≃ (R → R) compute-unit-continuation = equiv-precomp (inv-left-unit-law-function-type R) R
Computing continuation R
on the empty type
We have the equivalence
continuation R empty ≃ R.
module _ {l1 : Level} {R : UU l1} where compute-empty-continuation : continuation R empty ≃ R compute-empty-continuation = left-unit-law-Π-is-contr (universal-property-empty' R) ex-falso
External links
- continuation monad at Lab
Recent changes
- 2024-11-05. Fredrik Bakke and Egbert Rijke. Continuation modalities and Lawvere–Tierney topologies (#1157).