src/HOL/TPTP/MaSh_Eval.thy
author blanchet
Sat, 08 Dec 2012 00:48:50 +0100
changeset 50437 9762fe72936e
parent 50402 923f1e199f4f
child 50448 0a740d127187
permissions -rw-r--r--
store evaluation output in a file

(*  Title:      HOL/TPTP/MaSh_Eval.thy
    Author:     Jasmin Blanchette, TU Muenchen
*)

header {* MaSh Evaluation Driver *}

theory MaSh_Eval
imports Complex_Main
begin

ML_file "mash_eval.ML"

sledgehammer_params
  [provers = spass, max_relevant = 32, strict, dont_slice, type_enc = mono_native,
   lam_trans = combs_and_lifting, timeout = 15, dont_preplay, minimize]

declare [[sledgehammer_instantiate_inducts]]

ML {*
open MaSh_Eval
*}

ML {*
val do_it = false (* switch to "true" to generate the files *)
val params = Sledgehammer_Isar.default_params @{context} []
*}

ML {*
if do_it then
  evaluate_mash_suggestions @{context} params "/tmp/mash_suggestions"
      "/tmp/mash_eval.out"
else
  ()
*}

end