added interact flag to control mode of excursions;
authorwenzelm
Mon, 12 Sep 2005 12:11:17 +0200
changeset 17321 227f1f5c3959
parent 17320 e72f43c659f7
child 17322 781abf7011e6
added interact flag to control mode of excursions;
src/Pure/Isar/toplevel.ML
--- a/src/Pure/Isar/toplevel.ML	Sun Sep 11 20:02:51 2005 +0200
+++ b/src/Pure/Isar/toplevel.ML	Mon Sep 12 12:11:17 2005 +0200
@@ -37,6 +37,7 @@
   val pretty_state: bool -> state -> Pretty.T list
   val quiet: bool ref
   val debug: bool ref
+  val interact: bool ref
   val timing: bool ref
   val profiling: int ref
   val skip_proofs: bool ref
@@ -215,6 +216,7 @@
 
 val quiet = ref false;
 val debug = ref false;
+val interact = ref false;
 val timing = Output.timing;
 val profiling = ref 0;
 val skip_proofs = ref false;
@@ -574,7 +576,7 @@
 
 fun excur [] x = x
   | excur ((tr, pr) :: trs) (st, res) =
-      (case apply (! debug) tr st of
+      (case apply (! interact) tr st of
         SOME (st', NONE) =>
           excur trs (st', transform_error (fn () => pr st st' res) () handle exn =>
             raise EXCURSION_FAIL (exn, "Presentation failed\n" ^ at_command tr))