Theory Syntax
section ‹The $\lambda\mu$-calculus›
text‹More examples, as well as a call-by-value programming language built on
top of our formalisation, can be found in an associated Bitbucket repository~\<^cite>‹"bitbucket"›.›
theory Syntax
imports Main
begin
subsection ‹Syntax›
datatype type =
Iota
| Fun type type (infixr "→" 200)
text‹To deal with $\alpha$-equivalence, we use De Bruijn's nameless representation wherein each bound
variable is represented by a natural number, its index, that denotes the number of binders
that must be traversed to arrive at the one that binds the given variable.
Each free variable has an index that points into the top-level context, not enclosed in
any abstractions.›