aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/reduction.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-06-07 17:04:56 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-06-07 17:08:54 +0200
commit560b24f8eab0838fd6e01da8c4373f560020aadd (patch)
tree155efeee777cecabd7d2898da4689075129e43bc /kernel/reduction.ml
parent24a0df63c1844c6f2c69f9644a3059d668fd1e6f (diff)
Moving a Thread.yield in check_interrupt.
Diffstat (limited to 'kernel/reduction.ml')
-rw-r--r--kernel/reduction.ml14
1 files changed, 0 insertions, 14 deletions
diff --git a/kernel/reduction.ml b/kernel/reduction.ml
index c96371f26..6a8f3ddd7 100644
--- a/kernel/reduction.ml
+++ b/kernel/reduction.ml
@@ -265,15 +265,6 @@ let in_whnf (t,stk) =
| (FFlex _ | FProd _ | FEvar _ | FInd _ | FAtom _ | FRel _ | FProj _) -> true
| FLOCKED -> assert false
-let steps = ref 0
-
-let slave_process =
- let rec f = ref (fun () ->
- match !Flags.async_proofs_mode with
- | Flags.APonParallel n -> let b = n > 0 in f := (fun () -> b); !f ()
- | _ -> f := (fun () -> false); !f ()) in
- fun () -> !f ()
-
let unfold_projection infos p c =
if RedFlags.red_set infos.i_flags (RedFlags.fCONST p) then
(match try Some (lookup_projection p (info_env infos)) with Not_found -> None with
@@ -290,11 +281,6 @@ let rec ccnv cv_pb l2r infos lft1 lft2 term1 term2 cuniv =
(* Conversion between [lft1](hd1 v1) and [lft2](hd2 v2) *)
and eqappr cv_pb l2r infos (lft1,st1) (lft2,st2) cuniv =
Control.check_for_interrupt ();
- incr steps;
- if !steps = 10000 && slave_process () then begin
- Thread.yield ();
- steps := 0;
- end;
(* First head reduce both terms *)
let whd = whd_stack (infos_with_reds infos betaiotazeta) in
let rec whd_both (t1,stk1) (t2,stk2) =