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 55d7dcf2e..6bc449d5b 100644
--- a/toplevel/lemmas.mli
+++ b/toplevel/lemmas.mli
@@ -34,7 +34,7 @@ val start_proof_with_initialization :
(** A hook the next three functions pass to cook_proof *)
val set_save_hook : (Proof.proof -> unit) -> unit
-(** {6 Sect } *)
+(** {6 ... } *)
(** [save_named b] saves the current completed proof under the name it
was started; boolean [b] tells if the theorem is declared opaque; it
fails if the proof is not completed *)