aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/coqtop.ml
diff options
context:
space:
mode:
authorGravatar aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-08-09 14:53:14 +0000
committerGravatar aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-08-09 14:53:14 +0000
commitf6af94e119909d3a5dcc4624785f143c3dcdf73a (patch)
tree06517f9a8772f87d4a6d6e7608a460587bdafd3c /toplevel/coqtop.ml
parent9e6e9ccac3ac803229336cdef3b272ea7c857993 (diff)
Moved the declaration of "Classic" being the default proof mode to coqtop.ml so that the files in Init can benefit from the full-blown tactic language.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14392 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'toplevel/coqtop.ml')
-rw-r--r--toplevel/coqtop.ml2
1 files changed, 2 insertions, 0 deletions
diff --git a/toplevel/coqtop.ml b/toplevel/coqtop.ml
index 6f3b424e5..21ecdd5b0 100644
--- a/toplevel/coqtop.ml
+++ b/toplevel/coqtop.ml
@@ -315,6 +315,8 @@ let parse_args arglist =
let init arglist =
Sys.catch_break false; (* Ctrl-C is fatal during the initialisation *)
Lib.init();
+ (* Default Proofb Mode starts with an alternative default. *)
+ Goptions.set_string_option_value ["Default";"Proof";"Mode"] "Classic";
begin
try
let foreign_args = parse_args arglist in