From 75f569f35fbbbbab5a4629eaf3385335a3024e0b Mon Sep 17 00:00:00 2001 From: Emilio Jesus Gallego Arias Date: Sun, 11 Mar 2018 03:16:09 +0100 Subject: [vernac] Move `Quit` and `Drop` to the toplevel layer. This is a first step towards moving REPL-specific commands out of the core layers. In particular, we remove `Quit` and `Drop` from the core vernacular to specific toplevel-level parsing rules. --- toplevel/vernac.mli | 5 +++-- 1 file changed, 3 insertions(+), 2 deletions(-) (limited to 'toplevel/vernac.mli') diff --git a/toplevel/vernac.mli b/toplevel/vernac.mli index 51758642e..126954023 100644 --- a/toplevel/vernac.mli +++ b/toplevel/vernac.mli @@ -15,6 +15,7 @@ module State : sig doc : Stm.doc; sid : Stateid.t; proof : Proof.t option; + time : bool; } end @@ -23,10 +24,10 @@ end expected to handle and print errors in form of exceptions, however care is taken so the state machine is left in a consistent state. *) -val process_expr : time:bool -> state:State.t -> Vernacexpr.vernac_control CAst.t -> State.t +val process_expr : state:State.t -> Vernacexpr.vernac_control CAst.t -> State.t (** [load_vernac echo sid file] Loads [file] on top of [sid], will echo the commands if [echo] is set. Callers are expected to handle and print errors in form of exceptions. *) -val load_vernac : time:bool -> echo:bool -> check:bool -> interactive:bool -> +val load_vernac : echo:bool -> check:bool -> interactive:bool -> state:State.t -> string -> State.t -- cgit v1.2.3