src/HOL/Set.thy
changeset 26339 7825c83c9eff
parent 26150 f6bd8686b71e
child 26480 544cef16045b
--- a/src/HOL/Set.thy	Wed Mar 19 22:28:17 2008 +0100
+++ b/src/HOL/Set.thy	Wed Mar 19 22:47:35 2008 +0100
@@ -428,8 +428,8 @@
   Gives better instantiation for bound:
 *}
 
-ML_setup {*
-  change_claset (fn cs => cs addbefore ("bspec", datac @{thm bspec} 1))
+declaration {* fn _ =>
+  Classical.map_cs (fn cs => cs addbefore ("bspec", datac @{thm bspec} 1))
 *}
 
 lemma bexI [intro]: "P x ==> x:A ==> EX x:A. P x"
@@ -1031,9 +1031,11 @@
    ("Collect", [CollectD]), ("Inter", [InterD]), ("INTER", [INT_D])]
  *)
 
-ML_setup {*
+ML {*
   val mksimps_pairs = [("Ball", @{thms bspec})] @ mksimps_pairs;
-  change_simpset (fn ss => ss setmksimps (mksimps mksimps_pairs));
+*}
+declaration {* fn _ =>
+  Simplifier.map_ss (fn ss => ss setmksimps (mksimps mksimps_pairs))
 *}