aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/goal.mli
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.mli
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.mli')
-rw-r--r--proofs/goal.mli4
1 files changed, 2 insertions, 2 deletions
diff --git a/proofs/goal.mli b/proofs/goal.mli
index f887e8c66..4d3361b0e 100644
--- a/proofs/goal.mli
+++ b/proofs/goal.mli
@@ -133,6 +133,6 @@ 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 enter : (Environ.env -> Evd.evar_map -> Term.constr -> goal -> 'a) -> 'a sensitive
-val nf_enter : (Environ.env -> Evd.evar_map -> Environ.named_context_val -> Term.constr -> goal -> 'a) -> 'a sensitive
+val nf_enter : (Environ.env -> Evd.evar_map -> Term.constr -> goal -> 'a) -> 'a sensitive