aboutsummaryrefslogtreecommitdiff
path: root/engine
diff options
context:
space:
mode:
Diffstat (limited to 'engine')
-rw-r--r--engine/proofview.ml3
-rw-r--r--engine/proofview.mli3
2 files changed, 6 insertions, 0 deletions
diff --git a/engine/proofview.ml b/engine/proofview.ml
index de38104ecd..fd8512d73e 100644
--- a/engine/proofview.ml
+++ b/engine/proofview.ml
@@ -1032,6 +1032,9 @@ module Unsafe = struct
let mark_as_unresolvables p evs =
{ p with solution = mark_in_evm ~goal:false p.solution evs }
+ let update_sigma_env pv env =
+ { pv with solution = Evd.update_sigma_env pv.solution env }
+
end
module UnsafeRepr = Proof.Unsafe
diff --git a/engine/proofview.mli b/engine/proofview.mli
index d0a2b37a69..0f49d2f5d8 100644
--- a/engine/proofview.mli
+++ b/engine/proofview.mli
@@ -503,6 +503,9 @@ module Unsafe : sig
val undefined : Evd.evar_map -> Proofview_monad.goal_with_state list ->
Proofview_monad.goal_with_state list
+ (** [update_sigma_env] lifts [Evd.update_sigma_env] to the proofview *)
+ val update_sigma_env : proofview -> Environ.env -> proofview
+
end
(** This module gives access to the innards of the monad. Its use is