aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2018-03-04 16:30:15 +0100
committerGravatar Maxime Dénès <mail@maximedenes.fr>2018-03-04 16:30:15 +0100
commit346e73cef9e4e89c90f9f6f7011d54e3a0a35d96 (patch)
tree07ccc997e8e13eac81d2c2a7dc5d63284dfbdf77 /proofs
parented05111e048e864c63c2e21b8ebac675a80dc464 (diff)
parenta131ebf7b66e31dea7d8ccfb9706ad6d8f4a12e0 (diff)
Merge PR #6676: [proofview] goals come with a state
Diffstat (limited to 'proofs')
-rw-r--r--proofs/refine.ml2
1 files changed, 2 insertions, 0 deletions
diff --git a/proofs/refine.ml b/proofs/refine.ml
index 90276951b..73ed70a1a 100644
--- a/proofs/refine.ml
+++ b/proofs/refine.ml
@@ -73,6 +73,7 @@ let generic_refine ~typecheck f gl =
let sigma = Proofview.Goal.sigma gl in
let env = Proofview.Goal.env gl in
let concl = Proofview.Goal.concl gl in
+ let state = Proofview.Goal.state gl in
(** Save the [future_goals] state to restore them after the
refinement. *)
let prev_future_goals = Evd.future_goals sigma in
@@ -120,6 +121,7 @@ let generic_refine ~typecheck f gl =
(** Select the goals *)
let comb = CList.map_filter (Proofview.Unsafe.advance sigma) (CList.rev evs) in
let sigma = CList.fold_left Proofview.Unsafe.mark_as_goal sigma comb in
+ let comb = CList.map (fun x -> Proofview.goal_with_state x state) comb in
let trace () = Pp.(hov 2 (str"simple refine"++spc()++ Hook.get pr_constrv env sigma c)) in
Proofview.Trace.name_tactic trace (Proofview.tclUNIT v) >>= fun v ->
Proofview.Unsafe.tclSETENV (Environ.reset_context env) <*>