aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/vernac.mli
diff options
context:
space:
mode:
authorGravatar vgross <vgross@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-02-12 17:50:33 +0000
committerGravatar vgross <vgross@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-02-12 17:50:33 +0000
commitae0aa7b06204025bf22223823ab07e640e6cf094 (patch)
treedd9a85fd4525d9fa11fe67aae616677010564aba /toplevel/vernac.mli
parent088e63c756bafd5224016a079e9a1f43191a242c (diff)
Delineating a API for Coq inside toplevel/vernac.ml
Coq use case are mostly thoses : - parsing a char stream to get a vernac expr - evaluating a vernac expr with backtracking - turning a knob with a vernac expr, no backtracking - loading an entire file - compiling an entire file - backtracking (no clean API for this yet) - peeking Coq state info (no clean API for this yet) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12756 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'toplevel/vernac.mli')
-rw-r--r--toplevel/vernac.mli12
1 files changed, 4 insertions, 8 deletions
diff --git a/toplevel/vernac.mli b/toplevel/vernac.mli
index 4dff36e53..747c02afe 100644
--- a/toplevel/vernac.mli
+++ b/toplevel/vernac.mli
@@ -13,8 +13,8 @@
(* Read a vernac command on the specified input (parse only).
Raises [End_of_file] if EOF (or Ctrl-D) is reached. *)
-val parse_phrase : Pcoq.Gram.parsable * in_channel option ->
- Util.loc * Vernacexpr.vernac_expr
+val parse_sentence : Pcoq.Gram.parsable * in_channel option ->
+ Util.loc * Vernacexpr.vernac_expr
(* Reads and executes vernac commands from a stream.
The boolean [just_parsing] disables interpretation of commands. *)
@@ -23,6 +23,8 @@ exception DuringCommandInterp of Util.loc * exn
exception End_of_input
val just_parsing : bool ref
+val eval_expr : Util.loc * Vernacexpr.vernac_expr -> unit
+val eval_ctrl : Vernacexpr.vernac_expr -> unit
val raw_do_vernac : Pcoq.Gram.parsable -> unit
(* Set XML hooks *)
@@ -38,9 +40,3 @@ val load_vernac : bool -> string -> unit
(* Compile a vernac file, verbosely or not (f is assumed without .v suffix) *)
val compile : bool -> string -> unit
-
-(* Interpret a vernac AST *)
-
-val vernac_com :
- (Vernacexpr.vernac_expr -> unit) ->
- Util.loc * Vernacexpr.vernac_expr -> unit