src/HOL/Int.thy
changeset 61144 5e94dfead1c2
parent 61076 bdc1e2f0a86a
child 61169 4de9ff3ea29a
--- a/src/HOL/Int.thy	Wed Sep 09 14:47:41 2015 +0200
+++ b/src/HOL/Int.thy	Wed Sep 09 20:57:21 2015 +0200
@@ -775,9 +775,9 @@
 declaration \<open>K Int_Arith.setup\<close>
 
 simproc_setup fast_arith ("(m::'a::linordered_idom) < n" |
-  "(m::'a::linordered_idom) <= n" |
+  "(m::'a::linordered_idom) \<le> n" |
   "(m::'a::linordered_idom) = n") =
-  \<open>fn _ => fn ss => fn ct => Lin_Arith.simproc ss (Thm.term_of ct)\<close>
+  \<open>K Lin_Arith.simproc\<close>
 
 
 subsection\<open>More Inequality Reasoning\<close>