aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/proof_global.mli
diff options
context:
space:
mode:
Diffstat (limited to 'proofs/proof_global.mli')
-rw-r--r--proofs/proof_global.mli6
1 files changed, 4 insertions, 2 deletions
diff --git a/proofs/proof_global.mli b/proofs/proof_global.mli
index 5922075ec..9d7407010 100644
--- a/proofs/proof_global.mli
+++ b/proofs/proof_global.mli
@@ -64,12 +64,14 @@ type closed_proof =
(Entries.definition_entry list * lemma_possible_guards *
Decl_kinds.goal_kind * unit Tacexpr.declaration_hook)
-val close_proof : unit -> closed_proof
+(* Takes a function to add to the exceptions data relative to the
+ state in which the proof was built *)
+val close_proof : (exn -> exn) -> closed_proof
(* Intermediate step necessary to delegate the future.
* Both access the current proof state. The formes is supposed to be
* chained with a computation that completed the proof *)
-val return_proof : fix_exn:(exn -> exn) -> Entries.proof_output list
+val return_proof : unit -> Entries.proof_output list
val close_future_proof :
Entries.proof_output list Future.computation -> closed_proof