src/HOL/MicroJava/BV/Correct.ML
changeset 8032 1eaae1a2f8ff
parent 8023 3e5ddca613dd
child 8045 816f566c414f
--- a/src/HOL/MicroJava/BV/Correct.ML	Wed Nov 24 13:36:14 1999 +0100
+++ b/src/HOL/MicroJava/BV/Correct.ML	Thu Nov 25 12:01:28 1999 +0100
@@ -233,7 +233,7 @@
 (** hconf **)
 
 
-Goal "hp x = None \\<longrightarrow> G,hp\\<turnstile>\\<surd> \\<longrightarrow> G,hp\\<turnstile>obj\\<surd> \\<longrightarrow> G,hp(newref hp\\<mapsto>obj)\\<turnstile>\\<surd>";
+Goal "hp x = None \\<longrightarrow> G\\<turnstile>h hp\\<surd> \\<longrightarrow> G,hp\\<turnstile>obj\\<surd> \\<longrightarrow> G\\<turnstile>h hp(newref hp\\<mapsto>obj)\\<surd>";
 by (asm_full_simp_tac (simpset() addsplits [split_split] 
 				 addsimps [hconf_def]) 1);
  by (fast_tac (claset()addIs[oconf_imp_oconf_heap_newref] addss (simpset())) 1);
@@ -241,7 +241,7 @@
 
 
 Goal "map_of (fields (G, oT)) (F, D) = Some T \\<and> hp oloc = Some(oT,fs) \\<and> \
-\ G,hp\\<turnstile>v\\<Colon>\\<preceq>T \\<and> G,hp\\<turnstile>\\<surd> \\<longrightarrow> G,hp(oloc \\<mapsto> (oT, fs((F,D)\\<mapsto>v)))\\<turnstile>\\<surd>";
+\ G,hp\\<turnstile>v\\<Colon>\\<preceq>T \\<and> G\\<turnstile>h hp\\<surd> \\<longrightarrow> G\\<turnstile>h hp(oloc \\<mapsto> (oT, fs((F,D)\\<mapsto>v)))\\<surd>";
 by (asm_full_simp_tac (simpset() addsimps [hconf_def]) 1);
 by (fast_tac (claset() addIs 
         [oconf_imp_oconf_heap_update, oconf_imp_oconf_field_update]