src/HOL/MicroJava/Comp/CorrCompTp.thy
changeset 37456 0a1cc2675958
parent 35416 d8d7d1b785af
child 46226 e88e980ed735
equal deleted inserted replaced
37455:059ee3176686 37456:0a1cc2675958
  2370               (OK (Some (start_ST, start_LT C pTs mxl)))"
  2370               (OK (Some (start_ST, start_LT C pTs mxl)))"
  2371 apply (simp add: check_type_def wf_mhead_def start_ST_def start_LT_def)
  2371 apply (simp add: check_type_def wf_mhead_def start_ST_def start_LT_def)
  2372 apply (simp add: check_type_simps)
  2372 apply (simp add: check_type_simps)
  2373 apply (simp only: list_def)
  2373 apply (simp only: list_def)
  2374 apply (auto simp: err_def)
  2374 apply (auto simp: err_def)
  2375 apply (subgoal_tac "set (replicate mxl Err) \<subseteq>  {Err}")
       
  2376 apply blast
       
  2377 apply (rule subset_replicate)
       
  2378 done
  2375 done
  2379 
  2376 
  2380 
  2377 
  2381 lemma wt_method_comp_aux: "\<lbrakk>   bc' = bc @ [Return]; f' = (f \<box> nochangeST);
  2378 lemma wt_method_comp_aux: "\<lbrakk>   bc' = bc @ [Return]; f' = (f \<box> nochangeST);
  2382   bc_mt_corresp bc f sttp0 cG rT (1+length pTs+mxl) (length bc);
  2379   bc_mt_corresp bc f sttp0 cG rT (1+length pTs+mxl) (length bc);