src/HOL/MicroJava/JVM/JVMDefensive.thy
changeset 37406 982f3e02f3c4
parent 35417 47ee18b6ae32
child 53024 e0968e1f6fe9
--- a/src/HOL/MicroJava/JVM/JVMDefensive.thy	Fri Jun 11 17:14:01 2010 +0200
+++ b/src/HOL/MicroJava/JVM/JVMDefensive.thy	Fri Jun 11 17:14:01 2010 +0200
@@ -117,10 +117,10 @@
     | Normal s' \<Rightarrow> if check G s' then Normal (exec (G, s')) else TypeError"
 
 
-constdefs
+definition
   exec_all_d :: "jvm_prog \<Rightarrow> jvm_state type_error \<Rightarrow> jvm_state type_error \<Rightarrow> bool" 
-                   ("_ |- _ -jvmd-> _" [61,61,61]60)
-  "G |- s -jvmd-> t \<equiv>
+                   ("_ |- _ -jvmd-> _" [61,61,61]60) where
+  "G |- s -jvmd-> t \<longleftrightarrow>
          (s,t) \<in> ({(s,t). exec_d G s = TypeError \<and> t = TypeError} \<union>
                   {(s,t). \<exists>t'. exec_d G s = Normal (Some t') \<and> t = Normal t'})\<^sup>*"