Theory CK_Machine
theory CK_Machine
imports "HOL-Nominal.Nominal"
begin
text ‹
This theory establishes soundness and completeness for a CK-machine
with respect to a cbv-big-step semantics. The language includes
functions, recursion, booleans and numbers. In the soundness proof
the small-step cbv-reduction relation is used in order to get the
induction through. The type-preservation property is proved for the
machine and also for the small- and big-step semantics. Finally,
the progress property is proved for the small-step semantics.
The development is inspired by notes about context machines written
by Roshan James (Indiana University) and also by the lecture notes
written by Andy Pitts for his semantics course. See
🌐‹http://www.cs.indiana.edu/~rpjames/lm.pdf›
🌐‹https://www.cl.cam.ac.uk/teaching/2001/Semantics›
›