src/HOL/NanoJava/Example.thy
changeset 69597 ff784d5a5bfb
parent 68451 c34aa23a1fb6
child 80914 d97fdabd9e2b
equal deleted inserted replaced
69596:c8a2755bf220 69597:ff784d5a5bfb
   129   "heap s aa = None \<Longrightarrow> \<forall>v::val. s:v \<ge> n \<longrightarrow> hupd(aa\<mapsto>obj) s:v \<ge> n"
   129   "heap s aa = None \<Longrightarrow> \<forall>v::val. s:v \<ge> n \<longrightarrow> hupd(aa\<mapsto>obj) s:v \<ge> n"
   130 apply (induct n)
   130 apply (induct n)
   131 apply  auto
   131 apply  auto
   132 apply  (case_tac "aa=a")
   132 apply  (case_tac "aa=a")
   133 apply   auto
   133 apply   auto
   134 apply (tactic "smp_tac @{context} 1 1")
   134 apply (tactic "smp_tac \<^context> 1 1")
   135 apply (case_tac "aa=a")
   135 apply (case_tac "aa=a")
   136 apply  auto
   136 apply  auto
   137 done
   137 done
   138 
   138 
   139 
   139