aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/vernac.mli
diff options
context:
space:
mode:
authorGravatar aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-07-12 14:00:59 +0000
committerGravatar aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-07-12 14:00:59 +0000
commit944e0af31740558a38891498c375201dd61a1573 (patch)
treeac13ebedf006b0448257730062be5ecea1d64097 /toplevel/vernac.mli
parent2014b6b4153d034c4c0ee96de7b4fd20fb629492 (diff)
A new status Unsafe in Interface. Meant for commands such as Admitted.
Currently : - only Admitted uses the Unsafe return status - the status is ignored in coqtop - Coqide sees the status but apparently doesn't use it for colouring (I'm not sure why, but then again, it's not as if I understood coqide's code or anything) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15610 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'toplevel/vernac.mli')
-rw-r--r--toplevel/vernac.mli7
1 files changed, 4 insertions, 3 deletions
diff --git a/toplevel/vernac.mli b/toplevel/vernac.mli
index 924f2a65e..d76eb5d46 100644
--- a/toplevel/vernac.mli
+++ b/toplevel/vernac.mli
@@ -27,9 +27,10 @@ val just_parsing : bool ref
Backtrack stack (triggering a save of a frozen state and the generation
of a new state label). An example of state-preserving command is one coming
from the query panel of Coqide. *)
-
-val eval_expr : ?preserving:bool -> Loc.t * Vernacexpr.vernac_expr -> unit
-val raw_do_vernac : Pcoq.Gram.parsable -> unit
+(* spiwack: return value: [true] if safe (general case), [false] if
+ unsafe (like [Admitted]). *)
+val eval_expr : ?preserving:bool -> Loc.t * Vernacexpr.vernac_expr -> bool
+val raw_do_vernac : Pcoq.Gram.parsable -> bool
(** Set XML hooks *)
val set_xml_start_library : (unit -> unit) -> unit