src/HOL/MicroJava/BV/Correct.thy
changeset 13681 06cce9be31a4
parent 13052 3bf41c474a88
child 16417 9bc16273c2d4
--- a/src/HOL/MicroJava/BV/Correct.thy	Sat Oct 26 13:05:27 2002 +0200
+++ b/src/HOL/MicroJava/BV/Correct.thy	Sun Oct 27 23:34:02 2002 +0100
@@ -334,8 +334,7 @@
   "\<forall>rT C sig. 
   hp x = None \<longrightarrow> 
   correct_frames G hp phi rT sig frs \<longrightarrow>
-  G,hp \<turnstile> obj \<surd>
-  \<longrightarrow> correct_frames G (hp(x \<mapsto> obj)) phi rT sig frs"
+  correct_frames G (hp(x \<mapsto> obj)) phi rT sig frs"
 apply (induct frs)
  apply simp
 apply clarify