aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/proofview.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-07-14 00:01:28 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-07-14 00:01:28 +0200
commit99cee0e8d64567c6a89ab665c6e4dfd934674142 (patch)
tree478e1e7b4f6284cb90cda45d6e316115bb8eac44 /proofs/proofview.ml
parentc2b0ca88cbc4e874e7b3bd9b9f4c07477cb5b530 (diff)
Adding a delay to tclTIME.
Diffstat (limited to 'proofs/proofview.ml')
-rw-r--r--proofs/proofview.ml1
1 files changed, 1 insertions, 0 deletions
diff --git a/proofs/proofview.ml b/proofs/proofview.ml
index 6074a13d4..8df23a8bd 100644
--- a/proofs/proofview.ml
+++ b/proofs/proofview.ml
@@ -606,6 +606,7 @@ let tclTIME s t =
msg_info(str "Tactic call" ++ pr_opt str s ++ str " ran for " ++
System.fmt_time_difference t1 t2 ++ str " " ++ surround msg) in
let rec aux n t =
+ tclUNIT () >>= fun () ->
let tstart = System.get_time() in
Proof.split t >>= function
| Nil e ->