aboutsummaryrefslogtreecommitdiff
path: root/proofs
diff options
context:
space:
mode:
authorEnrico Tassi2020-08-19 11:17:49 +0200
committerEnrico Tassi2020-08-19 11:17:49 +0200
commitae38c38837e068721cc54d01570427aefdce49c5 (patch)
tree69adbd7922a6bc52f0758b8eca0095778f64c1d5 /proofs
parentdaed771ff18978dea536b277e00c0ca0149129ee (diff)
parent2edad4e3903ee77155f8b164c6cf6df49c897a27 (diff)
Merge PR #12725: Store evar identity instances in evarinfo / named_context_val
Ack-by: SkySkimmer Reviewed-by: gares
Diffstat (limited to 'proofs')
-rw-r--r--proofs/goal.ml6
1 files changed, 2 insertions, 4 deletions
diff --git a/proofs/goal.ml b/proofs/goal.ml
index beeaa60433..1c3aed8fc2 100644
--- a/proofs/goal.ml
+++ b/proofs/goal.ml
@@ -8,7 +8,6 @@
(* * (see LICENSE file for the text of the license) *)
(************************************************************************)
-open Util
open Pp
module NamedDecl = Context.Named.Declaration
@@ -58,12 +57,11 @@ module V82 = struct
goals are restored to their initial value after the evar is
created. *)
let prev_future_goals = Evd.save_future_goals evars in
+ let inst = EConstr.identity_subst_val hyps in
let (evars, evk) =
- Evarutil.new_pure_evar ~src:(Loc.tag Evar_kinds.GoalEvar) ~typeclass_candidate:false hyps evars concl
+ Evarutil.new_pure_evar ~src:(Loc.tag Evar_kinds.GoalEvar) ~typeclass_candidate:false ~identity:inst hyps evars concl
in
let evars = Evd.restore_future_goals evars prev_future_goals in
- let ctxt = Environ.named_context_of_val hyps in
- let inst = List.map (NamedDecl.get_id %> EConstr.mkVar) ctxt in
let ev = EConstr.mkEvar (evk,inst) in
(evk, ev, evars)