aboutsummaryrefslogtreecommitdiffhomepage
path: root/engine
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-12-06 08:58:50 +0100
committerGravatar Maxime Dénès <mail@maximedenes.fr>2018-03-08 21:58:26 +0100
commitd2c50bb29df8f0b23f7ee498abeda43a672fc688 (patch)
tree127379b1d724f5b7b76f2b0a48a942cc7552f35e /engine
parent866bad4e9cdaa6ff4419840f8c9980f770873176 (diff)
Proof engine: consider the pair principal and future goals as an entity.
Diffstat (limited to 'engine')
-rw-r--r--engine/evd.ml2
-rw-r--r--engine/evd.mli2
-rw-r--r--engine/proofview.ml2
3 files changed, 3 insertions, 3 deletions
diff --git a/engine/evd.ml b/engine/evd.ml
index 185cab101..e0453713e 100644
--- a/engine/evd.ml
+++ b/engine/evd.ml
@@ -946,7 +946,7 @@ let principal_future_goal evd = evd.principal_future_goal
let reset_future_goals evd =
{ evd with future_goals = [] ; principal_future_goal=None }
-let restore_future_goals evd gls pgl =
+let restore_future_goals evd (gls,pgl) =
{ evd with future_goals = gls ; principal_future_goal = pgl }
(**********************************************************)
diff --git a/engine/evd.mli b/engine/evd.mli
index 49c953f6d..49632d2e7 100644
--- a/engine/evd.mli
+++ b/engine/evd.mli
@@ -303,7 +303,7 @@ val reset_future_goals : evar_map -> evar_map
(** Clears the list of future goals (as well as the principal future
goal). Used by the [refine] primitive of the tactic engine. *)
-val restore_future_goals : evar_map -> Evar.t list -> Evar.t option -> evar_map
+val restore_future_goals : evar_map -> Evar.t list * Evar.t option -> evar_map
(** Sets the future goals (including the principal future goal) to a
previous value. Intended to be used after a local list of future
goals has been consumed. Used by the [refine] primitive of the
diff --git a/engine/proofview.ml b/engine/proofview.ml
index 8a844bbf5..4f8da5378 100644
--- a/engine/proofview.ml
+++ b/engine/proofview.ml
@@ -771,7 +771,7 @@ let with_shelf tac =
let gls' = Evd.future_goals sigma in
let fgoals = Evd.future_goals solution in
let pgoal = Evd.principal_future_goal solution in
- let sigma = Evd.restore_future_goals sigma fgoals pgoal in
+ let sigma = Evd.restore_future_goals sigma (fgoals,pgoal) in
(* Ensure we mark and return only unsolved goals *)
let gls' = undefined_evars sigma (CList.rev_append gls' gls) in
let sigma = CList.fold_left (mark_in_evm ~goal:false) sigma gls' in