aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/vernacentries.ml
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-12-19 12:00:44 +0100
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-12-19 12:00:57 +0100
commitab7d96a1d7c1bd44cf3bca5f593b947975117ed8 (patch)
tree346eac1f9ccddd701a6d160f493fd070bc84d09f /toplevel/vernacentries.ml
parent96906c2a1ba9426271a4048bfa8b3991db51c192 (diff)
Better doc and a few fixes for Proof using.
Diffstat (limited to 'toplevel/vernacentries.ml')
-rw-r--r--toplevel/vernacentries.ml3
1 files changed, 2 insertions, 1 deletions
diff --git a/toplevel/vernacentries.ml b/toplevel/vernacentries.ml
index 29ba18307..cd1dad694 100644
--- a/toplevel/vernacentries.ml
+++ b/toplevel/vernacentries.ml
@@ -848,7 +848,8 @@ let vernac_set_end_tac tac =
let vernac_set_used_variables e =
let tys =
- List.map fst (Proof.initial_goals (Proof_global.give_me_the_proof ())) in
+ List.map snd (Proof.initial_goals (Proof_global.give_me_the_proof ())) in
+ Pp.(msg_warning (prlist_with_sep spc Printer.pr_constr tys));
let l = Proof_using.process_expr (Global.env ()) e tys in
let vars = Environ.named_context (Global.env ()) in
List.iter (fun id ->