aboutsummaryrefslogtreecommitdiffhomepage
path: root/ide/coq.mli
diff options
context:
space:
mode:
Diffstat (limited to 'ide/coq.mli')
-rw-r--r--ide/coq.mli30
1 files changed, 18 insertions, 12 deletions
diff --git a/ide/coq.mli b/ide/coq.mli
index 9c8e27320..5ded2b573 100644
--- a/ide/coq.mli
+++ b/ide/coq.mli
@@ -15,10 +15,26 @@ open Evd
val version : unit -> string
+type reset_mark =
+ | ResetToId of Names.identifier
+ | ResetToState of Libnames.object_name
+
+type reset_info =
+ | NoReset
+ | ResetAtDecl of reset_mark * bool ref
+ | ResetAtSegmentStart of Names.identifier * bool ref
+ | ResetAtFrozenState of Libnames.object_name * bool ref
+
+val compute_reset_info : Vernacexpr.vernac_expr -> reset_info
+val reset_initial : unit -> unit
+val reset_to : reset_mark -> unit
+val reset_to_mod : identifier -> unit
+
val init : unit -> string list
-val interp : bool -> string -> Util.loc * Vernacexpr.vernac_expr
+val interp : bool -> string -> reset_info * (Util.loc * Vernacexpr.vernac_expr)
val interp_last : Util.loc * Vernacexpr.vernac_expr -> unit
-val interp_and_replace : string -> (Util.loc * Vernacexpr.vernac_expr) * string
+val interp_and_replace : string ->
+ (reset_info * (Util.loc * Vernacexpr.vernac_expr)) * string
val is_vernac_tactic_command : Vernacexpr.vernac_expr -> bool
val is_vernac_state_preserving_command : Vernacexpr.vernac_expr -> bool
@@ -42,16 +58,6 @@ val print_no_goal : unit -> string
val process_exn : exn -> string*(Util.loc option)
-type reset_info =
- | NoReset
- | ResetAtDecl of Names.identifier * bool ref
- | ResetAtSegmentStart of Names.identifier * bool ref
-
-val compute_reset_info : Vernacexpr.vernac_expr -> reset_info
-val reset_initial : unit -> unit
-val reset_to : identifier -> unit
-val reset_to_mod : identifier -> unit
-
val hyp_menu : hyp -> (string * string) list
val concl_menu : concl -> (string * string) list