src/HOL/Tools/etc/options
author blanchet
Wed, 18 Jun 2014 13:23:09 +0200
changeset 57272 fd539459a112
parent 57089 353652f47974
child 57431 02c408aed5ee
permissions -rw-r--r--
enabled MaSh by default -- set 'MaSh' to 'none' in Isabelle Plugin Options to disable

(* :mode=isabelle-options: *)

section {* Automatically tried tools *}

public option auto_time_start : real = 1.0
  -- "initial delay for automatically tried tools (seconds)"

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_methods : 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"


section "Miscellaneous Tools"

public option sledgehammer_provers : string = "e spass remote_vampire"
  -- "ATPs for Sledgehammer (separated by blanks)"

public option sledgehammer_timeout : int = 30
  -- "ATPs will be interrupted after this time (in seconds)"

public option z3_non_commercial : string = "unknown"
  -- "status of Z3 activation for non-commercial use (yes, no, unknown)"

public option MaSh : string = "sml"
  -- "machine learning engine to use by Sledgehammer (sml, sml_knn, sml_nb, py, none)"