aboutsummaryrefslogtreecommitdiffhomepage
path: root/vernac/lemmas.mli
diff options
context:
space:
mode:
authorGravatar Emilio Jesus Gallego Arias <e+git@x80.org>2017-11-24 09:56:55 +0100
committerGravatar Emilio Jesus Gallego Arias <e+git@x80.org>2017-11-29 14:07:34 +0100
commita41f8601655f69e71b621dba192342ed0e1f8ec2 (patch)
tree921861c20db73501b325befb8ce719f798abc30c /vernac/lemmas.mli
parentb23df225c7df7883af6ecfa921986cfb6fd3cd7c (diff)
[proof] [api] Rename proof types in preparation for functionalization.
In particular `Proof_global.t` will become a first class object for the upper parts of the system in a next commit.
Diffstat (limited to 'vernac/lemmas.mli')
-rw-r--r--vernac/lemmas.mli2
1 files changed, 1 insertions, 1 deletions
diff --git a/vernac/lemmas.mli b/vernac/lemmas.mli
index 1b1304db5..a4854b4a6 100644
--- a/vernac/lemmas.mli
+++ b/vernac/lemmas.mli
@@ -56,7 +56,7 @@ val standard_proof_terminator :
(** {6 ... } *)
(** A hook the next three functions pass to cook_proof *)
-val set_save_hook : (Proof.proof -> unit) -> unit
+val set_save_hook : (Proof.t -> unit) -> unit
val save_proof : ?proof:Proof_global.closed_proof -> Vernacexpr.proof_end -> unit