aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/goal.mli
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-09-03 21:43:45 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-09-03 22:46:03 +0200
commit8287733d5df1bd673a38e92f23c47e95d1bb7a91 (patch)
tree14185967d8e447ed1f3cfc51f3772bf24859bfaa /proofs/goal.mli
parent2c96be02dfa0a6169856a844dfc36b7f1053d0c5 (diff)
Putting back normalized goals when entering them.
This should allow tactics after a Goal.enter not to have to renormalize them uselessly.
Diffstat (limited to 'proofs/goal.mli')
-rw-r--r--proofs/goal.mli2
1 files changed, 2 insertions, 0 deletions
diff --git a/proofs/goal.mli b/proofs/goal.mli
index 535a2f2b1..f887e8c66 100644
--- a/proofs/goal.mli
+++ b/proofs/goal.mli
@@ -134,3 +134,5 @@ val refine_open_constr : Evd.open_constr -> subgoals sensitive
(* [enter] combines [env], [defs], [hyps] and [concl] in a single
primitive. *)
val enter : (Environ.env -> Evd.evar_map -> Environ.named_context_val -> Term.constr -> goal -> 'a) -> 'a sensitive
+
+val nf_enter : (Environ.env -> Evd.evar_map -> Environ.named_context_val -> Term.constr -> goal -> 'a) -> 'a sensitive