src/HOL/MicroJava/BV/BVNoTypeError.thy
changeset 14045 a34d89ce6097
parent 13822 bb5eda7416e5
child 14397 b3b15305a1c9
--- a/src/HOL/MicroJava/BV/BVNoTypeError.thy	Mon May 26 11:42:41 2003 +0200
+++ b/src/HOL/MicroJava/BV/BVNoTypeError.thy	Mon May 26 18:36:15 2003 +0200
@@ -299,9 +299,10 @@
         have "\<exists>D vs. hp (the_Addr v) = Some (D,vs) \<and> G \<turnstile> D \<preceq>C C" 
           by (auto dest!: non_np_objD)
       }
-      ultimately show ?thesis using Getfield field class stk hconf
+      ultimately show ?thesis using Getfield field class stk hconf wf
         apply clarsimp
-        apply (fastsimp dest!: hconfD widen_cfs_fields [OF _ _ wf] oconf_objD)
+        apply (fastsimp intro: wf_prog_ws_prog
+	  dest!: hconfD widen_cfs_fields oconf_objD)
         done
     next
       case (Putfield F C)