moved some rat functions to library.ML
authornipkow
Sun, 07 Aug 2005 12:30:45 +0200
changeset 17029 7839e85fc246
parent 17028 a497f621bfd4
child 17030 ab8c7fbf235b
moved some rat functions to library.ML
src/Provers/Arith/fast_lin_arith.ML
--- a/src/Provers/Arith/fast_lin_arith.ML	Sun Aug 07 12:28:10 2005 +0200
+++ b/src/Provers/Arith/fast_lin_arith.ML	Sun Aug 07 12:30:45 2005 +0200
@@ -167,8 +167,6 @@
   | elim_eqns(ineqs,Lineq(i,Eq,cs,_)) = (i,true,cs)::(~i,true,map ~ cs)::ineqs
   | elim_eqns(ineqs,Lineq(i,Lt,cs,_)) = (i,false,cs)::ineqs;
 
-val rat0 = rat_of_int 0;
-
 (* PRE: ex[v] must be 0! *)
 fun eval (ex:rat list) v (a:IntInf.int,le,cs:IntInf.int list) =
   let val rs = map rat_of_intinf cs
@@ -178,9 +176,6 @@
    Instead this swap is taken into account in ratrelmin2.
 *)
 
-fun ratge0 r = fst(rep_rat r) >= 0;
-fun ratle(r,s) = ratge0(ratadd(s,ratneg r));
-
 fun ratrelmin2(x as (r,ler),y as (s,les)) =
   if r=s then (r, (not ler) andalso (not les)) else if ratle(r,s) then x else y;
 fun ratrelmax2(x as (r,ler),y as (s,les)) =