aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/goal.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-09-04 21:03:55 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-09-04 21:06:14 +0200
commitba801cd1c9866f39782279e22ceab956c4efd5c6 (patch)
tree99cc8bc1b8ad61de84a03a8eed6110f68f9bca33 /proofs/goal.ml
parent7057e7e9ab1160fc0e176182b6e71f720784715a (diff)
Ensuring the invariant that hypotheses and named context of the environment of
Proofview goals coincide by always using the named context and discarding the hypotheses.
Diffstat (limited to 'proofs/goal.ml')
-rw-r--r--proofs/goal.ml6
1 files changed, 3 insertions, 3 deletions
diff --git a/proofs/goal.ml b/proofs/goal.ml
index 6cdd315f8..fe8096db1 100644
--- a/proofs/goal.ml
+++ b/proofs/goal.ml
@@ -244,12 +244,12 @@ let refine_open_constr c =
let enter f = (); fun env rdefs gl info ->
let sigma = !rdefs in
- f env sigma (Evd.evar_hyps info) (Evd.evar_concl info) gl
+ f env sigma (Evd.evar_concl info) gl
let nf_enter f = (); fun env rdefs gl info ->
let sigma = !rdefs in
if gl.cache == sigma then
- f env sigma (Evd.evar_hyps info) (Evd.evar_concl info) gl
+ f env sigma (Evd.evar_concl info) gl
else
let info = Evarutil.nf_evar_info sigma info in
let sigma = Evd.add sigma gl.content info in
@@ -257,7 +257,7 @@ let nf_enter f = (); fun env rdefs gl info ->
let () = rdefs := sigma in
let hyps = Evd.evar_hyps info in
let env = Environ.reset_with_named_context hyps env in
- f env sigma hyps (Evd.evar_concl info) gl
+ f env sigma (Evd.evar_concl info) gl
(* Layer to implement v8.2 tactic engine ontop of the new architecture.
Types are different from what they used to be due to a change of the