aboutsummaryrefslogtreecommitdiffhomepage
path: root/engine
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2018-02-21 23:37:26 +0100
committerGravatar Maxime Dénès <mail@maximedenes.fr>2018-03-08 21:58:32 +0100
commit29aa2d94b253dad0ade8c877fd7f46b8537a5847 (patch)
treef16dde502481bd1438b5b48bda63014a475927ac /engine
parent81f14b203ac8476623ed6567844df452a1646a60 (diff)
A comment in Proofview.with_shelf.
Diffstat (limited to 'engine')
-rw-r--r--engine/proofview.ml2
1 files changed, 2 insertions, 0 deletions
diff --git a/engine/proofview.ml b/engine/proofview.ml
index 53b3cdd9b..22271dd02 100644
--- a/engine/proofview.ml
+++ b/engine/proofview.ml
@@ -768,6 +768,8 @@ let with_shelf tac =
tac >>= fun ans ->
Pv.get >>= fun npv ->
let { shelf = gls; solution = sigma } = npv in
+ (* The pending future goals are necessarily coming from V82.tactic *)
+ (* and thus considered as to shelve, as in Proof.run_tactic *)
let gls' = Evd.future_goals sigma in
let fgoals = Evd.save_future_goals solution in
let sigma = Evd.restore_future_goals sigma fgoals in