author | paulson |
Wed, 05 Aug 1998 10:57:25 +0200 | |
changeset 5253 | 82a5ca6290aa |
parent 5183 | 89f162de39cf |
child 8029 | 05446a898852 |
permissions | -rw-r--r-- |
(* Title: HOL/IMP/Com.thy ID: $Id$ Author: Heiko Loetzbeyer & Robert Sandner & Tobias Nipkow, TUM Copyright 1994 TUM Semantics of arithmetic and boolean expressions Syntax of commands *) Com = Datatype + types val loc state = "loc => val" aexp = "state => val" bexp = state => bool arities loc,val :: term datatype com = SKIP | ":=" loc aexp (infixl 60) | Semi com com ("_; _" [60, 60] 10) | Cond bexp com com ("IF _ THEN _ ELSE _" 60) | While bexp com ("WHILE _ DO _" 60) end