src/HOL/Decision_Procs/Dense_Linear_Order.thy
changeset 63198 c583ca33076a
parent 61586 5197a2ecb658
child 63201 f151704c08e4
--- a/src/HOL/Decision_Procs/Dense_Linear_Order.thy	Tue May 31 19:51:01 2016 +0200
+++ b/src/HOL/Decision_Procs/Dense_Linear_Order.thy	Tue May 31 21:54:10 2016 +0200
@@ -923,7 +923,7 @@
         val cr = dest_frac c
         val clt = Thm.dest_fun2 ct
         val cz = Thm.dest_arg ct
-        val neg = cr </ Rat.zero
+        val neg = cr < Rat.zero
         val cthp = Simplifier.rewrite ctxt
                (Thm.apply @{cterm "Trueprop"}
                   (if neg then Thm.apply (Thm.apply clt c) cz
@@ -946,7 +946,7 @@
         val cr = dest_frac c
         val clt = Thm.dest_fun2 ct
         val cz = Thm.dest_arg ct
-        val neg = cr </ Rat.zero
+        val neg = cr < Rat.zero
         val cthp = Simplifier.rewrite ctxt
                (Thm.apply @{cterm "Trueprop"}
                   (if neg then Thm.apply (Thm.apply clt c) cz
@@ -968,7 +968,7 @@
         val cr = dest_frac c
         val clt = Thm.cterm_of ctxt (Const (@{const_name ord_class.less}, T --> T --> @{typ bool}))
         val cz = Thm.dest_arg ct
-        val neg = cr </ Rat.zero
+        val neg = cr < Rat.zero
         val cthp = Simplifier.rewrite ctxt
                (Thm.apply @{cterm "Trueprop"}
                   (if neg then Thm.apply (Thm.apply clt c) cz
@@ -993,7 +993,7 @@
         val cr = dest_frac c
         val clt = Thm.cterm_of ctxt (Const (@{const_name ord_class.less}, T --> T --> @{typ bool}))
         val cz = Thm.dest_arg ct
-        val neg = cr </ Rat.zero
+        val neg = cr < Rat.zero
         val cthp = Simplifier.rewrite ctxt
                (Thm.apply @{cterm "Trueprop"}
                   (if neg then Thm.apply (Thm.apply clt c) cz