aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/proof_global.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2015-10-30 19:32:28 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2015-10-30 19:35:49 +0100
commit35afb42a6bb30634d2eb77a32002ed473633b5f4 (patch)
tree464483d6ef42aa817793297c5ac146d4b68307d8 /proofs/proof_global.ml
parentbf1eef119ef8f0e6a2ae4b66165d6e22c1ce9236 (diff)
parentb49c80406f518d273056b2143f55e23deeea2813 (diff)
Merge branch 'v8.5'
Diffstat (limited to 'proofs/proof_global.ml')
-rw-r--r--proofs/proof_global.ml6
1 files changed, 6 insertions, 0 deletions
diff --git a/proofs/proof_global.ml b/proofs/proof_global.ml
index e036ae3a1..1e0de05dd 100644
--- a/proofs/proof_global.ml
+++ b/proofs/proof_global.ml
@@ -703,3 +703,9 @@ let copy_terminators ~src ~tgt =
assert(List.length src = List.length tgt);
List.map2 (fun op p -> { p with terminator = op.terminator }) src tgt
+let update_global_env () =
+ with_current_proof (fun _ p ->
+ Proof.in_proof p (fun sigma ->
+ let tac = Proofview.Unsafe.tclEVARS (Evd.update_sigma_env sigma (Global.env ())) in
+ let (p,(status,info)) = Proof.run_tactic (Global.env ()) tac p in
+ (p, ())))