src/HOL/IMP/Com.thy
author nipkow
Sat, 27 Apr 1996 18:47:31 +0200
changeset 1696 e84bff5c519b
parent 1481 03f096efa26d
child 5183 89f162de39cf
permissions -rw-r--r--
A completely new version of IMP.

(*  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 = Arith +

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