(* * Copyright 2016, Data61, CSIRO * * This software may be distributed and modified according to the terms of * the BSD 2-Clause license. Note that NO WARRANTY is provided. * See "LICENSE_BSD2.txt" for details. * * @TAG(DATA61_BSD) *) section ‹COMPLX small-step semantics› theory SmallStep imports Language begin text ‹The procedure environment› type_synonym ('s,'p,'f) body = "'p ⇒ ('s,'p,'f) com option" text ‹State types›