src/HOL/Tools/etc/options
author wenzelm
Sat, 13 Jul 2013 14:11:48 +0200
changeset 52645 e8c1c5612677
parent 52639 df830310e550
child 52651 5adb5c69af97
permissions -rw-r--r--
clarified some default options;

(* :mode=isabelle-options: *)

section {* Isabelle/HOL proof tools *}

public option auto_time_limit : real = 2.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 = true
  -- "run Quickcheck automatically"

public option auto_solve_direct : bool = true
  -- "run solve_direct automatically"