aboutsummaryrefslogtreecommitdiffhomepage
path: root/ide/coqide.mli
diff options
context:
space:
mode:
Diffstat (limited to 'ide/coqide.mli')
-rw-r--r--ide/coqide.mli18
1 files changed, 12 insertions, 6 deletions
diff --git a/ide/coqide.mli b/ide/coqide.mli
index de9eb0238..f6f5b616f 100644
--- a/ide/coqide.mli
+++ b/ide/coqide.mli
@@ -6,10 +6,7 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(* The CoqIde main module. The following function [start] will parse the
- command line, initialize the load path, load the input
- state, load the files given on the command line, load the ressource file,
- produce the output state if any, and finally will launch the interface. *)
+(** * The CoqIde main module *)
(** The arguments that will be passed to coqtop. No quoting here, since
no /bin/sh when using create_process instead of open_process. *)
@@ -22,9 +19,18 @@ val set_coqtop_path : string list -> string list
(** Ask coqtop the remaining options it doesn't recognize *)
val process_argv : string list -> string list
+(** Prepare the widgets, load the given files in tabs *)
+val main : string list -> unit
+
+(** The function doing the actual loading of a file. *)
val do_load : string -> unit
-val crash_save : int -> unit
+(** Set coqide to ignore Ctrl-C, while launching [crash_save] and
+ exiting for others received signals *)
val ignore_break : unit -> unit
+
+(** Emergency saving of opened files as "foo.v.crashcoqide",
+ and exit (if the integer isn't 127). *)
+val crash_save : int -> unit
+
val check_for_geoproof_input : unit -> unit
-val main : string list -> unit