aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/lemmas.mli
diff options
context:
space:
mode:
Diffstat (limited to 'toplevel/lemmas.mli')
-rw-r--r--toplevel/lemmas.mli2
1 files changed, 1 insertions, 1 deletions
diff --git a/toplevel/lemmas.mli b/toplevel/lemmas.mli
index 6bc449d5b..b75d56999 100644
--- a/toplevel/lemmas.mli
+++ b/toplevel/lemmas.mli
@@ -29,7 +29,7 @@ val start_proof_com : goal_kind ->
val start_proof_with_initialization :
goal_kind -> (bool * lemma_possible_guards * tactic list option) option ->
(identifier * (types * (int * Impargs.manual_explicitation list))) list ->
- declaration_hook -> unit
+ int list option -> declaration_hook -> unit
(** A hook the next three functions pass to cook_proof *)
val set_save_hook : (Proof.proof -> unit) -> unit