src/HOL/Product_Type.thy
changeset 26480 544cef16045b
parent 26358 d6a508c16908
child 26588 d83271bfaba5
--- a/src/HOL/Product_Type.thy	Sat Mar 29 19:13:58 2008 +0100
+++ b/src/HOL/Product_Type.thy	Sat Mar 29 19:14:00 2008 +0100
@@ -57,7 +57,7 @@
   this rule directly --- it loops!
 *}
 
-ML_setup {*
+ML {*
   val unit_eq_proc =
     let val unit_meta_eq = mk_meta_eq @{thm unit_eq} in
       Simplifier.simproc @{theory} "unit_eq" ["x::unit"]
@@ -323,7 +323,7 @@
 
 lemmas split_tupled_all = split_paired_all unit_all_eq2
 
-ML_setup {*
+ML {*
   (* replace parameters of product type by individual component parameters *)
   val safe_full_simp_tac = generic_simp_tac true (true, false, false);
   local (* filtering with exists_paired_all is an essential optimization *)
@@ -429,7 +429,7 @@
   split_beta}.
 *}
 
-ML_setup {*
+ML {*
 
 local
   val cond_split_eta_ss = HOL_basic_ss addsimps [thm "cond_split_eta"]