src/HOL/IMPP/Com.thy
changeset 23746 a455e69c31cc
parent 19803 aa2581752afb
child 27362 a6dc1769fdda
--- a/src/HOL/IMPP/Com.thy	Wed Jul 11 11:13:08 2007 +0200
+++ b/src/HOL/IMPP/Com.thy	Wed Jul 11 11:14:51 2007 +0200
@@ -48,32 +48,29 @@
 
 
 (* Well-typedness: all procedures called must exist *)
-consts WTs :: "com set"
-syntax WT  :: "com => bool"
-translations "WT c" == "c : WTs"
 
-inductive WTs intros
+inductive WT  :: "com => bool" where
 
     Skip:    "WT SKIP"
 
-    Assign:  "WT (X :== a)"
+  | Assign:  "WT (X :== a)"
 
-    Local:   "WT c ==>
+  | Local:   "WT c ==>
               WT (LOCAL Y := a IN c)"
 
-    Semi:    "[| WT c0; WT c1 |] ==>
+  | Semi:    "[| WT c0; WT c1 |] ==>
               WT (c0;; c1)"
 
-    If:      "[| WT c0; WT c1 |] ==>
+  | If:      "[| WT c0; WT c1 |] ==>
               WT (IF b THEN c0 ELSE c1)"
 
-    While:   "WT c ==>
+  | While:   "WT c ==>
               WT (WHILE b DO c)"
 
-    Body:    "body pn ~= None ==>
+  | Body:    "body pn ~= None ==>
               WT (BODY pn)"
 
-    Call:    "WT (BODY pn) ==>
+  | Call:    "WT (BODY pn) ==>
               WT (X:=CALL pn(a))"
 
 inductive_cases WTs_elim_cases: