aboutsummaryrefslogtreecommitdiff
path: root/stm
diff options
context:
space:
mode:
authorJim Fehrle2020-12-17 15:04:36 -0800
committerJim Fehrle2021-01-13 15:24:23 -0800
commit3da2dbe9728ae7f5b1860a8e3a6c458e6d976f84 (patch)
treed9c17317be7ff621361ad1663b43efa5779dff39 /stm
parentb8a3ebaa9695596f062298f5913ae4f4debb0124 (diff)
Avoid using "subgoals" in the UI, it means the same as "goals"
Diffstat (limited to 'stm')
-rw-r--r--stm/partac.ml4
1 files changed, 2 insertions, 2 deletions
diff --git a/stm/partac.ml b/stm/partac.ml
index 8232b017f9..6143ac450b 100644
--- a/stm/partac.ml
+++ b/stm/partac.ml
@@ -125,7 +125,7 @@ end = struct (* {{{ *)
str" existentials remain unsolved: " ++ prlist (Termops.pr_existential_key sigma) (Evar.Set.elements evars))
)
with e when CErrors.noncritical e ->
- RespError (CErrors.print e ++ spc() ++ str "(for subgoal "++int r_goalno ++ str ")")
+ RespError (CErrors.print e ++ spc() ++ str "(for goal "++int r_goalno ++ str ")")
let name_of_task { t_name } = t_name
let name_of_request { r_name } = r_name
@@ -163,7 +163,7 @@ let enable_par ~nworkers = ComTactic.set_par_implementation
let open TacTask in
let results = (Proof.data p).Proof.goals |> CList.map_i (fun i g ->
let g_solution, t_assign =
- Future.create_delegate ~name:(Printf.sprintf "subgoal %d" i)
+ Future.create_delegate ~name:(Printf.sprintf "goal %d" i)
(fun x -> x) in
TaskQueue.enqueue_task queue
~cancel_switch:(ref false)