aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/pfedit.mli
diff options
context:
space:
mode:
authorGravatar Arnaud Spiwack <arnaud@spiwack.net>2013-11-27 18:41:09 +0100
committerGravatar Arnaud Spiwack <arnaud@spiwack.net>2013-12-04 14:14:33 +0100
commitf1a2c15b7a7d7edfd4b4b379ed0bde8b1f5deb7b (patch)
tree7f29564ddfa4d1bf2d4a06b6dd212cc3ef3beaff /proofs/pfedit.mli
parenteaa9c147f1801c363635a5be4e0258e0de1ab02e (diff)
Factoring(continued).
This commit removes the hook.
Diffstat (limited to 'proofs/pfedit.mli')
-rw-r--r--proofs/pfedit.mli14
1 files changed, 6 insertions, 8 deletions
diff --git a/proofs/pfedit.mli b/proofs/pfedit.mli
index 9762d415f..c3d0c9053 100644
--- a/proofs/pfedit.mli
+++ b/proofs/pfedit.mli
@@ -62,7 +62,7 @@ type lemma_possible_guards = Proof_global.lemma_possible_guards
val start_proof :
Id.t -> goal_kind -> named_context_val -> constr ->
?init_tac:unit Proofview.tactic ->
- unit declaration_hook -> Proof_global.proof_terminator -> unit
+ Proof_global.proof_terminator -> unit
(** {6 ... } *)
(** [cook_proof opacity] turns the current proof (assumed completed) into
@@ -70,16 +70,14 @@ val start_proof :
it fails if there is no current proof of if it is not completed;
it also tells if the guardness condition has to be inferred. *)
-val cook_this_proof : (Proof.proof -> unit) ->
+val cook_this_proof :
Proof_global.proof_object ->
(Id.t *
- (Entries.definition_entry * goal_kind *
- unit declaration_hook Ephemeron.key))
+ (Entries.definition_entry * goal_kind))
-val cook_proof : (Proof.proof -> unit) ->
+val cook_proof : unit ->
(Id.t *
- (Entries.definition_entry * goal_kind *
- unit declaration_hook Ephemeron.key))
+ (Entries.definition_entry * goal_kind))
(** {6 ... } *)
(** [get_pftreestate ()] returns the current focused pending proof.
@@ -100,7 +98,7 @@ val get_current_goal_context : unit -> Evd.evar_map * env
(** [current_proof_statement] *)
val current_proof_statement :
- unit -> Id.t * goal_kind * types * unit declaration_hook Ephemeron.key
+ unit -> Id.t * goal_kind * types
(** {6 ... } *)
(** [get_current_proof_name ()] return the name of the current focused