(* * 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 ‹The COMPLX Syntax› theory Language imports Main begin subsection ‹The Core Language› text ‹We use a shallow embedding of boolean expressions as well as assertions as sets of states. › type_synonym 's bexp = "'s set" type_synonym 's assn = "'s set"