src/HOL/Tools/etc/options
changeset 52639 df830310e550
child 52645 e8c1c5612677
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Tools/etc/options	Fri Jul 12 23:45:05 2013 +0200
@@ -0,0 +1,22 @@
+(* :mode=isabelle-options: *)
+
+section {* Isabelle/HOL proof tools *}
+
+public option auto_time_limit : real = 4.0
+  -- "time limit for automatically tried tools (seconds > 0)"
+
+public option auto_nitpick : bool = false
+  -- "run Nitpick automatically"
+
+public option auto_sledgehammer : bool = false
+  -- "run Sledgehammer automatically"
+
+public option auto_try0 : bool = false
+  -- "try standard proof methods automatically"
+
+public option auto_quickcheck : bool = false
+  -- "run Quickcheck automatically"
+
+public option auto_solve_direct : bool = false
+  -- "run solve_direct automatically"
+