src/HOL/Induct/Com.thy
changeset 24824 b7866aea0815
parent 24178 4ff1dc2aa18d
child 26806 40b411ec05aa
--- a/src/HOL/Induct/Com.thy	Wed Oct 03 19:36:05 2007 +0200
+++ b/src/HOL/Induct/Com.thy	Wed Oct 03 19:49:33 2007 +0200
@@ -11,20 +11,18 @@
 theory Com imports Main begin
 
 typedecl loc
-
 types  state = "loc => nat"
-       n2n2n = "nat => nat => nat"
 
 datatype
   exp = N nat
       | X loc
-      | Op n2n2n exp exp
+      | Op "nat => nat => nat" exp exp
       | valOf com exp          ("VALOF _ RESULTIS _"  60)
 and
   com = SKIP
-      | ":="  loc exp          (infixl  60)
-      | Semi  com com          ("_;;_"  [60, 60] 60)
-      | Cond  exp com com      ("IF _ THEN _ ELSE _"  60)
+      | Assign loc exp         (infixl ":=" 60)
+      | Semi com com           ("_;;_"  [60, 60] 60)
+      | Cond exp com com       ("IF _ THEN _ ELSE _"  60)
       | While exp com          ("WHILE _ DO _"  60)