src/HOL/Hyperreal/hypreal_arith0.ML
changeset 13462 56610e2ba220
parent 12018 ec054019c910
child 14331 8dbbb7cf3637
--- a/src/HOL/Hyperreal/hypreal_arith0.ML	Tue Aug 06 11:20:47 2002 +0200
+++ b/src/HOL/Hyperreal/hypreal_arith0.ML	Tue Aug 06 11:22:05 2002 +0200
@@ -44,11 +44,6 @@
      "(i <= j) & (k < l)  ==> i + k < j + (l::hypreal)",
      "(i < j) & (k < l)   ==> i + k < j + (l::hypreal)"];
 
-val hypreal_arith_simproc_pats =
-  map (fn s => Thm.read_cterm (Theory.sign_of (the_context ()))
-       (s, HOLogic.boolT))
-      ["(m::hypreal) < n", "(m::hypreal) <= n", "(m::hypreal) = n"];
-
 fun cvar(th,_ $ (_ $ _ $ var)) = cterm_of (#sign(rep_thm th)) var;
 
 val hypreal_mult_mono_thms =
@@ -59,8 +54,10 @@
 
 in
 
-val fast_hypreal_arith_simproc = mk_simproc
-  "fast_hypreal_arith" hypreal_arith_simproc_pats Fast_Arith.lin_arith_prover;
+val fast_hypreal_arith_simproc =
+  Simplifier.simproc (Theory.sign_of (the_context ()))
+    "fast_hypreal_arith" ["(m::hypreal) < n", "(m::hypreal) <= n", "(m::hypreal) = n"]
+    Fast_Arith.lin_arith_prover;
 
 val hypreal_arith_setup =
  [Fast_Arith.map_data (fn {add_mono_thms, mult_mono_thms, inj_thms, lessD, simpset} =>