aboutsummaryrefslogtreecommitdiff
path: root/toplevel
diff options
context:
space:
mode:
authorHugo Herbelin2019-10-11 21:04:51 +0200
committerHugo Herbelin2019-10-11 21:04:51 +0200
commite8d0b5a8856a695dc3f6a28e2d305c095ef50c19 (patch)
tree2afd2098b100e5432f5c3c907166d85610196316 /toplevel
parentf41cb3d7206155c8ad7321ff76e58bf5bd079c89 (diff)
parent04105f0430cad4e8d018ab47efccf79bf8511a32 (diff)
Merge PR #10489: Fix output for "Printing Dependent Evars Line"
Reviewed-by: Zimmi48 Reviewed-by: ejgallego Ack-by: hendriktews Reviewed-by: herbelin Ack-by: mattam82
Diffstat (limited to 'toplevel')
-rw-r--r--toplevel/coqloop.ml12
1 files changed, 11 insertions, 1 deletions
diff --git a/toplevel/coqloop.ml b/toplevel/coqloop.ml
index 07466d641e..1f319d2bfd 100644
--- a/toplevel/coqloop.ml
+++ b/toplevel/coqloop.ml
@@ -405,7 +405,17 @@ let rec vernac_loop ~state =
| Some (VernacShowGoal {gid; sid}) ->
let proof = Stm.get_proof ~doc:state.doc (Stateid.of_int sid) in
- Feedback.msg_notice (Printer.pr_goal_emacs ~proof gid sid);
+ let goal = Printer.pr_goal_emacs ~proof gid sid in
+ let evars =
+ match proof with
+ | None -> mt()
+ | Some p ->
+ let gl = (Evar.unsafe_of_int gid) in
+ let { Proof.sigma } = Proof.data p in
+ try Printer.print_dependent_evars (Some gl) sigma [ gl ]
+ with Not_found -> mt()
+ in
+ Feedback.msg_notice (v 0 (goal ++ evars));
vernac_loop ~state
| None ->