src/HOL/MicroJava/Comp/CorrCompTp.thy
changeset 22780 41162a270151
parent 21312 1d39091a3208
child 23022 9872ef956276
equal deleted inserted replaced
22779:9ac0ca736969 22780:41162a270151
   979 
   979 
   980 lemma bc_mt_corresp_zero [simp]: "\<lbrakk> length (mt_of (f sttp)) = length bc; start_sttp_resp f\<rbrakk>
   980 lemma bc_mt_corresp_zero [simp]: "\<lbrakk> length (mt_of (f sttp)) = length bc; start_sttp_resp f\<rbrakk>
   981   \<Longrightarrow> bc_mt_corresp bc f sttp cG rT mxr 0"
   981   \<Longrightarrow> bc_mt_corresp bc f sttp cG rT mxr 0"
   982 apply (simp add: bc_mt_corresp_def start_sttp_resp_def split_beta)
   982 apply (simp add: bc_mt_corresp_def start_sttp_resp_def split_beta)
   983 apply (erule disjE)
   983 apply (erule disjE)
   984 apply (simp add: max_ssize_def max_of_list_def ssize_sto_def split_beta)
   984 apply (simp add: max_ssize_def max_of_list_def ssize_sto_def split: prod.split)
   985 apply (intro strip)
   985 apply (intro strip)
   986 apply (simp add: start_sttp_resp_cons_def split_beta)
   986 apply (simp add: start_sttp_resp_cons_def split_beta)
   987 apply (drule_tac x=sttp in spec, erule exE)
   987 apply (drule_tac x=sttp in spec, erule exE)
   988 apply simp
   988 apply simp
   989 apply (rule check_type_mono, assumption)
   989 apply (rule check_type_mono, assumption)
   990 apply (simp add: max_ssize_def max_of_list_def ssize_sto_def max_def split_beta)
   990 apply (simp add: max_ssize_def max_of_list_def ssize_sto_def max_def split: prod.split)
   991 done
   991 done
   992 
   992 
   993   (* ********************************************************************** *)
   993   (* ********************************************************************** *)
   994 
   994 
   995 
   995