src/HOL/NSA/HyperDef.thy
changeset 38715 6513ea67d95d
parent 37765 26bdfb7b680b
child 42463 f270e3e18be5
--- a/src/HOL/NSA/HyperDef.thy	Wed Aug 25 18:19:04 2010 +0200
+++ b/src/HOL/NSA/HyperDef.thy	Wed Aug 25 18:36:22 2010 +0200
@@ -349,7 +349,7 @@
       @{thm star_of_number_of}, @{thm star_of_add}, @{thm star_of_minus},
       @{thm star_of_diff}, @{thm star_of_mult}]
   #> Lin_Arith.add_inj_const (@{const_name "StarDef.star_of"}, @{typ "real \<Rightarrow> hypreal"})
-  #> Simplifier.map_ss (fn simpset => simpset addsimprocs [Simplifier.simproc @{theory}
+  #> Simplifier.map_ss (fn simpset => simpset addsimprocs [Simplifier.simproc_global @{theory}
       "fast_hypreal_arith" ["(m::hypreal) < n", "(m::hypreal) <= n", "(m::hypreal) = n"]
       (K Lin_Arith.simproc)]))
 *}