src/HOL/MicroJava/Comp/CorrCompTp.thy
changeset 23315 df3a7e9ebadb
parent 23022 9872ef956276
child 24078 04b28c723d43
equal deleted inserted replaced
23314:6894137e854a 23315:df3a7e9ebadb
   520 
   520 
   521 
   521 
   522 lemma pc_succs_shift: "pc'\<in>set (succs i (pc'' + n))
   522 lemma pc_succs_shift: "pc'\<in>set (succs i (pc'' + n))
   523  \<Longrightarrow> ((pc' - n) \<in>set (succs i pc''))"
   523  \<Longrightarrow> ((pc' - n) \<in>set (succs i pc''))"
   524 apply (induct i)
   524 apply (induct i)
   525 apply (arith|simp)+
   525 apply simp_all
       
   526 apply arith
   526 done
   527 done
   527 
   528 
   528 
   529 
   529 lemma pc_succs_le: "\<lbrakk> pc' \<in> set (succs i (pc'' + n));   
   530 lemma pc_succs_le: "\<lbrakk> pc' \<in> set (succs i (pc'' + n));   
   530   \<forall> b. ((i = (Goto b) \<or> i=(Ifcmpeq b)) \<longrightarrow> 0 \<le> (int pc'' + b)) \<rbrakk> 
   531   \<forall> b. ((i = (Goto b) \<or> i=(Ifcmpeq b)) \<longrightarrow> 0 \<le> (int pc'' + b)) \<rbrakk> 
   531   \<Longrightarrow> n \<le> pc'"
   532   \<Longrightarrow> n \<le> pc'"
   532 apply (induct i)
   533 apply (induct i)
   533 apply (arith|simp)+
   534 apply simp_all
       
   535 apply arith
   534 done
   536 done
   535 
   537 
   536 
   538 
   537 (**********************************************************************)
   539 (**********************************************************************)
   538 
   540