src/Provers/Arith/fast_lin_arith.ML
changeset 17496 26535df536ae
parent 17325 d9d50222808e
child 17515 830bc15e692c
--- a/src/Provers/Arith/fast_lin_arith.ML	Tue Sep 20 08:20:22 2005 +0200
+++ b/src/Provers/Arith/fast_lin_arith.ML	Tue Sep 20 08:21:49 2005 +0200
@@ -278,7 +278,7 @@
   if n = 1 then i
   else if n = 0 andalso ty = Lt then sys_error "multiply_ineq"
   else if n < 0 andalso (ty=Le orelse ty=Lt) then sys_error "multiply_ineq"
-  else Lineq(n * k,ty,map (apl(n,op * )) l,Multiplied(n,just));
+  else Lineq (n * k, ty, map (curry (op *) n) l, Multiplied (n, just));
 
 (* ------------------------------------------------------------------------- *)
 (* Add together (in)equations.                                               *)
@@ -317,7 +317,7 @@
   case ty  of Eq => k <> 0 | Le => k > 0 | Lt => k >= 0;
 
 fun calc_blowup (l:IntInf.int list) =
-  let val (p,n) = List.partition (apl(0,op<)) (List.filter (apl(0,op<>)) l)
+  let val (p,n) = List.partition (curry (op <) 0) (List.filter (curry (op <>) 0) l)
   in (length p) * (length n) end;
 
 (* ------------------------------------------------------------------------- *)
@@ -538,11 +538,11 @@
   in a ^ " = " ^ s end;
 
 fun print_ex sds =
-  tracing o
-  apl("Counter example:\n",op ^) o
-  commas o
-  map print_atom o
-  apl(sds, op ~~);
+  curry (op ~~) sds
+  #> map print_atom
+  #> commas
+  #> curry (op ^) "Counter example:\n"
+  #> tracing;
 
 fun trace_ex(sg,params,atoms,discr,n,hist:history) =
   if null hist then ()