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:11:25 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-09-04 23:28:24 +0200
commitd55921dbacdc21a640b80482fb32188fa99febe7 (patch)
treeee63c7af7cdbe749bb46b4d354ff3a1661898d80 /proofs/goal.ml
parentba801cd1c9866f39782279e22ceab956c4efd5c6 (diff)
Only using filtered hyps in Goal.enter.
This was probably a bug. A user-side code should never be able to observe the difference between filtered and unfiltered hypotheses.
Diffstat (limited to 'proofs/goal.ml')
-rw-r--r--proofs/goal.ml4
1 files changed, 2 insertions, 2 deletions
diff --git a/proofs/goal.ml b/proofs/goal.ml
index fe8096db1..dc55c8179 100644
--- a/proofs/goal.ml
+++ b/proofs/goal.ml
@@ -141,7 +141,7 @@ type 'a sensitive =
as an optimisation (it shouldn't change during the evaluation). *)
let eval t env defs gl =
let info = content defs gl in
- let env = Environ.reset_with_named_context (Evd.evar_hyps info) env in
+ let env = Environ.reset_with_named_context (Evd.evar_filtered_hyps info) env in
let rdefs = ref defs in
let r = t env rdefs gl info in
( r , !rdefs )
@@ -255,7 +255,7 @@ let nf_enter f = (); fun env rdefs gl info ->
let sigma = Evd.add sigma gl.content info in
let gl = { gl with cache = sigma } in
let () = rdefs := sigma in
- let hyps = Evd.evar_hyps info in
+ let hyps = Evd.evar_filtered_hyps info in
let env = Environ.reset_with_named_context hyps env in
f env sigma (Evd.evar_concl info) gl