aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-11-27 11:07:45 +0100
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-11-27 16:06:54 +0100
commitdf8779378c3ea30f90b11204828c3a33513b9e3d (patch)
tree525a8406e70e13ea9e63489f2692d1e736ac200a
parent72f471f42d7825b9ef370fb5a64acbd155d9140e (diff)
async_queries_* merged with async_proofs_*
-rw-r--r--lib/flags.ml1
-rw-r--r--lib/flags.mli1
-rw-r--r--stm/stm.ml4
-rw-r--r--toplevel/coqtop.ml3
4 files changed, 3 insertions, 6 deletions
diff --git a/lib/flags.ml b/lib/flags.ml
index bcd7c59d7..31b40dc53 100644
--- a/lib/flags.ml
+++ b/lib/flags.ml
@@ -56,7 +56,6 @@ let async_proofs_n_workers = ref 1
let async_proofs_n_tacworkers = ref 2
let async_proofs_private_flags = ref None
let async_proofs_always_delegate = ref false
-let async_queries_always_delegate = ref false
let async_proofs_never_reopen_branch = ref false
let async_proofs_flags_for_workers = ref []
let async_proofs_worker_id = ref "master"
diff --git a/lib/flags.mli b/lib/flags.mli
index 716d04163..0c922ebb4 100644
--- a/lib/flags.mli
+++ b/lib/flags.mli
@@ -25,7 +25,6 @@ val async_proofs_private_flags : string option ref
val async_proofs_is_worker : unit -> bool
val async_proofs_is_master : unit -> bool
val async_proofs_always_delegate : bool ref
-val async_queries_always_delegate : bool ref
val async_proofs_never_reopen_branch : bool ref
val async_proofs_flags_for_workers : string list ref
val async_proofs_worker_id : string ref
diff --git a/stm/stm.ml b/stm/stm.ml
index 2d1d8aefe..35c723913 100644
--- a/stm/stm.ml
+++ b/stm/stm.ml
@@ -1500,7 +1500,7 @@ end = struct (* {{{ *)
QueryTask.({ QueryTask.t_where = prev; t_for = id; t_what = q }) switch
let init () = queue := Some (TaskQueue.create
- (if !Flags.async_queries_always_delegate then 1 else 0))
+ (if !Flags.async_proofs_always_delegate then 1 else 0))
end (* }}} *)
@@ -1969,7 +1969,7 @@ let process_transaction ?(newtip=Stateid.fresh ()) ~tty verbose c (loc, expr) =
assert(Stateid.equal report_id Stateid.dummy);
let id = VCS.new_node ~id:newtip () in
let queue =
- if !Flags.async_queries_always_delegate then `QueryQueue (ref false)
+ if !Flags.async_proofs_always_delegate then `QueryQueue (ref false)
else `MainQueue in
VCS.commit id (Cmd { cast = x; cids = []; cqueue = queue });
Backtrack.record (); if w == VtNow then finish (); `Ok
diff --git a/toplevel/coqtop.ml b/toplevel/coqtop.ml
index 255544d47..5bf8cfb3b 100644
--- a/toplevel/coqtop.ml
+++ b/toplevel/coqtop.ml
@@ -465,8 +465,7 @@ let parse_args arglist =
|"-toploop" -> toploop := Some (next ())
(* Options with zero arg *)
- |"-async-queries-always-delegate" ->
- Flags.async_queries_always_delegate := true;
+ |"-async-queries-always-delegate"
|"-async-proofs-always-delegate" ->
Flags.async_proofs_always_delegate := true;
|"-async-proofs-never-reopen-branch" ->