src/ZF/OrdQuant.thy
changeset 26339 7825c83c9eff
parent 24893 b8ef7afe3a6b
child 26480 544cef16045b
--- a/src/ZF/OrdQuant.thy	Wed Mar 19 22:28:17 2008 +0100
+++ b/src/ZF/OrdQuant.thy	Wed Mar 19 22:47:35 2008 +0100
@@ -362,7 +362,9 @@
     atomize ([("OrdQuant.oall", [@{thm ospec}]),("OrdQuant.rall", [@{thm rspec}])]@
                  ZF_conn_pairs,
              ZF_mem_pairs);
-change_simpset (fn ss => ss setmksimps (map mk_eq o Ord_atomize o gen_all));
+*}
+declaration {* fn _ =>
+  Simplifier.map_ss (fn ss => ss setmksimps (map mk_eq o Ord_atomize o gen_all))
 *}
 
 text {* Setting up the one-point-rule simproc *}