aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/proof.mli
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-01-26 13:24:04 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-01-26 18:39:41 +0100
commitc7a0568967a8a6e40888a2106b9b59325f2f09a5 (patch)
tree131f69969a4f5b0f49029479c9724acee3a371fc /proofs/proof.mli
parentd6bcc6ebe4f65d0555414851f7e4fb6fa1fb22a4 (diff)
Adding a printer for Proof.proof reflecting the focusing layout.
This is a modest contribution serving before all the purpose of displaying the focus stack and the shelf and give_up list. It does not print the sigma (while it could). Any improvements are welcome.
Diffstat (limited to 'proofs/proof.mli')
-rw-r--r--proofs/proof.mli2
1 files changed, 2 insertions, 0 deletions
diff --git a/proofs/proof.mli b/proofs/proof.mli
index 5053fc7fb..8dc165e72 100644
--- a/proofs/proof.mli
+++ b/proofs/proof.mli
@@ -182,6 +182,8 @@ val in_proof : proof -> (Evd.evar_map -> 'a) -> 'a
focused goals. *)
val unshelve : proof -> proof
+val pr_proof : proof -> Pp.std_ppcmds
+
(*** Compatibility layer with <=v8.2 ***)
module V82 : sig
val subgoals : proof -> Goal.goal list Evd.sigma