aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--ide/command_windows.mli22
-rw-r--r--ide/coq_tactics.mli12
-rw-r--r--ide/coqide.mli16
-rw-r--r--ide/ideutils.mli47
-rw-r--r--ide/preferences.mli55
5 files changed, 152 insertions, 0 deletions
diff --git a/ide/command_windows.mli b/ide/command_windows.mli
new file mode 100644
index 000000000..64800d359
--- /dev/null
+++ b/ide/command_windows.mli
@@ -0,0 +1,22 @@
+(***********************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * INRIA-Rocquencourt & LRI-CNRS-Orsay *)
+(* \VV/ *************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(***********************************************************************)
+
+(* $Id$ *)
+
+class command_window :
+ unit ->
+ object
+ method new_command : ?command:string -> ?term:string -> unit -> unit
+ method window : GWindow.window
+ end
+
+val main : unit -> unit
+
+val command_window : unit -> command_window
+
+
diff --git a/ide/coq_tactics.mli b/ide/coq_tactics.mli
new file mode 100644
index 000000000..6ed9e7998
--- /dev/null
+++ b/ide/coq_tactics.mli
@@ -0,0 +1,12 @@
+(***********************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * INRIA-Rocquencourt & LRI-CNRS-Orsay *)
+(* \VV/ *************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(***********************************************************************)
+
+(* $Id$ *)
+
+val tactics : string list
+
diff --git a/ide/coqide.mli b/ide/coqide.mli
new file mode 100644
index 000000000..b5ffba051
--- /dev/null
+++ b/ide/coqide.mli
@@ -0,0 +1,16 @@
+(***********************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * INRIA-Rocquencourt & LRI-CNRS-Orsay *)
+(* \VV/ *************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(***********************************************************************)
+
+(* $Id$ *)
+
+(* 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. *)
+
+val start : unit -> unit
diff --git a/ide/ideutils.mli b/ide/ideutils.mli
new file mode 100644
index 000000000..2e98c0594
--- /dev/null
+++ b/ide/ideutils.mli
@@ -0,0 +1,47 @@
+(***********************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * INRIA-Rocquencourt & LRI-CNRS-Orsay *)
+(* \VV/ *************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(***********************************************************************)
+
+(* $Id$ *)
+
+val async : ('a -> unit) -> 'a -> unit
+val browse : string -> unit
+val browse_keyword : string -> unit
+val byte_offset_to_char_offset : string -> int -> int
+val clear_stdout : unit -> unit
+val debug : bool ref
+val disconnect_revert_timer : unit -> unit
+val disconnect_auto_save_timer : unit -> unit
+val do_convert : string -> string
+val find_tag_limits : GText.tag -> GText.iter -> GText.iter * GText.iter
+val find_tag_start : GText.tag -> GText.iter -> GText.iter
+val find_tag_stop : GText.tag -> GText.iter -> GText.iter
+val get_insert : < get_iter_at_mark : [> `INSERT] -> 'a; .. > -> 'a
+
+val is_char_start : char -> bool
+
+val lib_ide : string
+val my_stat : string -> Unix.stats option
+
+val prerr_endline : string -> unit
+val prerr_string : string -> unit
+val print_id : 'a -> unit
+
+val process_pending : unit -> unit
+val read_stdout : unit -> string
+val revert_timer : GMain.Timeout.id option ref
+val auto_save_timer : GMain.Timeout.id option ref
+val select_file :
+ title:string ->
+ ?dir:string ref -> ?filename:string -> unit -> string option
+val set_highlight_timer : (unit -> 'a) -> unit
+val try_convert : string -> string
+val try_export : string -> string -> bool
+val stock_to_widget : ?size:Gtk.Tags.icon_size -> GtkStock.id -> GObj.widget
+
+open Format
+val print_list : (formatter -> 'a -> unit) -> formatter -> 'a list -> unit
diff --git a/ide/preferences.mli b/ide/preferences.mli
new file mode 100644
index 000000000..055d621d4
--- /dev/null
+++ b/ide/preferences.mli
@@ -0,0 +1,55 @@
+(***********************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * INRIA-Rocquencourt & LRI-CNRS-Orsay *)
+(* \VV/ *************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(***********************************************************************)
+
+(* $Id$ *)
+
+type pref =
+ {
+ mutable cmd_coqc : string;
+ mutable cmd_make : string;
+ mutable cmd_coqmakefile : string;
+ mutable cmd_coqdoc : string;
+
+ mutable global_auto_revert : bool;
+ mutable global_auto_revert_delay : int;
+
+ mutable auto_save : bool;
+ mutable auto_save_delay : int;
+ mutable auto_save_name : string * string;
+
+ mutable automatic_tactics : (string * string) list;
+ mutable cmd_print : string;
+
+ mutable modifier_for_navigation : Gdk.Tags.modifier list;
+ mutable modifier_for_templates : Gdk.Tags.modifier list;
+ mutable modifier_for_tactics : Gdk.Tags.modifier list;
+ mutable modifiers_valid : Gdk.Tags.modifier list;
+
+ mutable cmd_browse : string * string;
+
+ mutable text_font : Pango.font_description;
+
+ mutable doc_url : string;
+ mutable library_url : string;
+
+ mutable show_toolbar : bool;
+ mutable window_width : int;
+ mutable window_height : int;
+
+ }
+
+val save_pref : unit -> unit
+val load_pref : unit -> unit
+
+val current : pref ref
+
+val configure : unit -> unit
+
+val change_font : ( Pango.font_description -> unit) ref
+val show_toolbar : (bool -> unit) ref
+val resize_window : (unit -> unit) ref