src/HOL/IMP/Procs.thy
author kleing
Sat, 13 Aug 2011 11:57:13 +0200
changeset 44177 b4b5cbca2519
parent 43158 686fa0a0696e
child 45212 e87feee00a4c
permissions -rw-r--r--
IMP/Util distinguishes between sets and functions again; imported only where used.

header "Extensions and Variations of IMP"

theory Procs imports BExp begin

subsection "Procedures and Local Variables"

datatype
  com = SKIP 
      | Assign name aexp         ("_ ::= _" [1000, 61] 61)
      | Semi   com  com          ("_;/ _"  [60, 61] 60)
      | If     bexp com com     ("(IF _/ THEN _/ ELSE _)"  [0, 0, 61] 61)
      | While  bexp com         ("(WHILE _/ DO _)"  [0, 61] 61)
      | Var    name com         ("(1{VAR _;;/ _})")
      | Proc   name com com     ("(1{PROC _ = _;;/ _})")
      | CALL   name

definition "test_com =
{VAR ''x'';;
 ''x'' ::= N 0;
 {PROC ''p'' = ''x'' ::= Plus (V ''x'') (V ''x'');;
  {PROC ''q'' = CALL ''p'';;
   {VAR ''x'';;
    ''x'' ::= N 5;
    {PROC ''p'' = ''x'' ::= Plus (V ''x'') (N 1);;
     CALL ''q''; ''y'' ::= V ''x''}}}}}"

end