aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/goal.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-03-11 18:28:50 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-03-19 13:34:23 +0100
commit27e4cb0e99497997c9d019607b578685a71b5944 (patch)
tree86d82e2c48f62293a33e22b46eb80cbfaabebf04 /proofs/goal.ml
parent0ed5686e28f93d5832ce08c6728ff1c4bc5b431c (diff)
Adding phantom types to discriminate normalized goals, and adding a way to
observe non-normalized goals.
Diffstat (limited to 'proofs/goal.ml')
-rw-r--r--proofs/goal.ml5
1 files changed, 1 insertions, 4 deletions
diff --git a/proofs/goal.ml b/proofs/goal.ml
index b0fded289..64eeb69d9 100644
--- a/proofs/goal.ml
+++ b/proofs/goal.ml
@@ -375,10 +375,7 @@ let defs _ rdefs _ _ =
let enter f = (); fun env rdefs gl info ->
let sigma = !rdefs in
- let concl = Reductionops.nf_evar sigma (Evd.evar_concl info) in
- let map_nf c = Reductionops.nf_evar sigma c in
- let hyps = Environ.map_named_val map_nf (Evd.evar_hyps info) in
- f env sigma hyps concl gl
+ f env sigma (Evd.evar_hyps info) (Evd.evar_concl info) gl
(*** Conversion in goals ***)