src/HOL/Bali/WellForm.thy
changeset 52037 837211662fb8
parent 51717 9e7d1c139569
child 55518 1ddb2edf5ceb
equal deleted inserted replaced
52036:1aa2e40df9ff 52037:837211662fb8
  2256       by (cases emh type: prod) (auto dest: accmethd_SomeD)
  2256       by (cases emh type: prod) (auto dest: accmethd_SomeD)
  2257   qed
  2257   qed
  2258 qed
  2258 qed
  2259 declare split_paired_All [simp] split_paired_Ex [simp]
  2259 declare split_paired_All [simp] split_paired_Ex [simp]
  2260 setup {* map_theory_claset (fn ctxt => ctxt addSbefore ("split_all_tac", split_all_tac)) *}
  2260 setup {* map_theory_claset (fn ctxt => ctxt addSbefore ("split_all_tac", split_all_tac)) *}
  2261 setup {* map_theory_simpset (fn ctxt => ctxt addloop' ("split_all_tac", split_all_tac)) *}
  2261 setup {* map_theory_simpset (fn ctxt => ctxt addloop ("split_all_tac", split_all_tac)) *}
  2262 
  2262 
  2263 (* Tactical version *)
  2263 (* Tactical version *)
  2264 (*
  2264 (*
  2265 lemma dynamic_mheadsD: "  
  2265 lemma dynamic_mheadsD: "  
  2266  \<lbrakk>emh \<in> mheads G S statT sig; wf_prog G; class G dynC = Some y;  
  2266  \<lbrakk>emh \<in> mheads G S statT sig; wf_prog G; class G dynC = Some y;  
  2425              simp add: is_acc_type_def
  2425              simp add: is_acc_type_def
  2426     )
  2426     )
  2427 done
  2427 done
  2428 declare split_paired_All [simp] split_paired_Ex [simp]
  2428 declare split_paired_All [simp] split_paired_Ex [simp]
  2429 setup {* map_theory_claset (fn ctxt => ctxt addSbefore ("split_all_tac", split_all_tac)) *}
  2429 setup {* map_theory_claset (fn ctxt => ctxt addSbefore ("split_all_tac", split_all_tac)) *}
  2430 setup {* map_theory_simpset (fn ctxt => ctxt addloop' ("split_all_tac", split_all_tac)) *}
  2430 setup {* map_theory_simpset (fn ctxt => ctxt addloop ("split_all_tac", split_all_tac)) *}
  2431 
  2431 
  2432 lemma ty_expr_is_type: 
  2432 lemma ty_expr_is_type: 
  2433 "\<lbrakk>E\<turnstile>e\<Colon>-T; wf_prog (prg E)\<rbrakk> \<Longrightarrow> is_type (prg E) T"
  2433 "\<lbrakk>E\<turnstile>e\<Colon>-T; wf_prog (prg E)\<rbrakk> \<Longrightarrow> is_type (prg E) T"
  2434 by (auto dest!: wt_is_type)
  2434 by (auto dest!: wt_is_type)
  2435 lemma ty_var_is_type: 
  2435 lemma ty_var_is_type: