aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/proof_global.mli
diff options
context:
space:
mode:
authorGravatar Pierre Courtieu <Pierre.Courtieu@cnam.fr>2015-01-08 16:59:47 +0100
committerGravatar Pierre Courtieu <Pierre.Courtieu@cnam.fr>2015-01-08 16:59:57 +0100
commitb92fff621cce1576c93fab9276fb41ea85e10982 (patch)
treed6e0c1964b274c9b00339452d77468f48ebe2794 /proofs/proof_global.mli
parent448bf4529c5766e98367345076d00e64e25db7bf (diff)
Fixed and extend bullet related info/error messages. + doc.
Had to put some hook in the handler of Proofview.NoSuchgoals. Documentation updated. CHANGE updated.
Diffstat (limited to 'proofs/proof_global.mli')
-rw-r--r--proofs/proof_global.mli9
1 files changed, 6 insertions, 3 deletions
diff --git a/proofs/proof_global.mli b/proofs/proof_global.mli
index c9a812c4c..f9f67235b 100644
--- a/proofs/proof_global.mli
+++ b/proofs/proof_global.mli
@@ -151,11 +151,13 @@ module Bullet : sig
type t = Vernacexpr.bullet
(** A [behavior] is the data of a put function which
- is called when a bullet prefixes a tactic, together
- with a name to identify it. *)
+ is called when a bullet prefixes a tactic, a suggest function
+ suggesting the right bullet to use on a given proof, together
+ with a name to identify the behavior. *)
type behavior = {
name : string;
- put : Proof.proof -> t -> Proof.proof
+ put : Proof.proof -> t -> Proof.proof;
+ suggest: Proof.proof -> string option
}
(** A registered behavior can then be accessed in Coq
@@ -172,6 +174,7 @@ module Bullet : sig
(** Handles focusing/defocusing with bullets:
*)
val put : Proof.proof -> t -> Proof.proof
+ val suggest : Proof.proof -> string option
end