src/HOL/Bali/Eval.thy
changeset 13462 56610e2ba220
parent 13384 a34e38154413
child 13601 fd3e3d6b37b2
--- a/src/HOL/Bali/Eval.thy	Tue Aug 06 11:20:47 2002 +0200
+++ b/src/HOL/Bali/Eval.thy	Tue Aug 06 11:22:05 2002 +0200
@@ -894,7 +894,7 @@
   fun pred (_ $ (Const ("Pair",_) $ _ $ 
       (Const ("Pair", _) $ _ $ (Const ("Pair", _) $ x $ _ ))) $ _ ) = is_Inj x
 in
-  make_simproc name lhs pred (thm name)
+  cond_simproc name lhs pred (thm name)
 end
 
 val eval_expr_proc =eval_fun "expr" "In1l" "\<exists>v.  w=In1 v   \<and> G\<turnstile>s \<midarrow>t-\<succ>v \<rightarrow> s'"
@@ -989,7 +989,7 @@
      (Const ("Pair", _) $ x $ _) $ _ ) $ _)) = is_None x
 in
   val eval_no_abrupt_proc = 
-  make_simproc "eval_no_abrupt" "G\<turnstile>(x,s) \<midarrow>e\<succ>\<rightarrow> (w,Norm s')" pred 
+  cond_simproc "eval_no_abrupt" "G\<turnstile>(x,s) \<midarrow>e\<succ>\<rightarrow> (w,Norm s')" pred 
           (thm "eval_no_abrupt")
 end;
 Addsimprocs [eval_no_abrupt_proc]
@@ -1017,7 +1017,7 @@
        x))) $ _ ) = is_Some x
 in
   val eval_abrupt_proc = 
-  make_simproc "eval_abrupt" 
+  cond_simproc "eval_abrupt" 
                "G\<turnstile>(Some xc,s) \<midarrow>e\<succ>\<rightarrow> (w,s')" pred (thm "eval_abrupt")
 end;
 Addsimprocs [eval_abrupt_proc]