src/HOL/Bali/WellForm.thy
changeset 52037 837211662fb8
parent 51717 9e7d1c139569
child 55518 1ddb2edf5ceb
--- a/src/HOL/Bali/WellForm.thy	Thu May 16 15:21:12 2013 +0200
+++ b/src/HOL/Bali/WellForm.thy	Thu May 16 17:39:38 2013 +0200
@@ -2258,7 +2258,7 @@
 qed
 declare split_paired_All [simp] split_paired_Ex [simp]
 setup {* map_theory_claset (fn ctxt => ctxt addSbefore ("split_all_tac", split_all_tac)) *}
-setup {* map_theory_simpset (fn ctxt => ctxt addloop' ("split_all_tac", split_all_tac)) *}
+setup {* map_theory_simpset (fn ctxt => ctxt addloop ("split_all_tac", split_all_tac)) *}
 
 (* Tactical version *)
 (*
@@ -2427,7 +2427,7 @@
 done
 declare split_paired_All [simp] split_paired_Ex [simp]
 setup {* map_theory_claset (fn ctxt => ctxt addSbefore ("split_all_tac", split_all_tac)) *}
-setup {* map_theory_simpset (fn ctxt => ctxt addloop' ("split_all_tac", split_all_tac)) *}
+setup {* map_theory_simpset (fn ctxt => ctxt addloop ("split_all_tac", split_all_tac)) *}
 
 lemma ty_expr_is_type: 
 "\<lbrakk>E\<turnstile>e\<Colon>-T; wf_prog (prg E)\<rbrakk> \<Longrightarrow> is_type (prg E) T"