diff -r 02bdd591eb8f -r 4ad62c5f9f88 src/HOL/TPTP/ATP_Problem_Import.thy --- a/src/HOL/TPTP/ATP_Problem_Import.thy Fri Apr 27 15:24:37 2012 +0200 +++ b/src/HOL/TPTP/ATP_Problem_Import.thy Fri Apr 27 15:24:37 2012 +0200 @@ -6,7 +6,7 @@ theory ATP_Problem_Import imports Complex_Main TPTP_Interpret uses "sledgehammer_tactics.ML" - "atp_problem_import.ML" + ("atp_problem_import.ML") begin ML {* Proofterm.proofs := 0 *} @@ -14,8 +14,14 @@ declare [[show_consts]] (* for Refute *) declare [[smt_oracle]] +declare [[unify_search_bound = 60]] +declare [[unify_trace_bound = 60]] + +use "atp_problem_import.ML" + (* -ML {* ATP_Problem_Import.isabelle_tptp_file 300 "$TPTP/Problems/PUZ/PUZ107^5.p" *} +ML {* ATP_Problem_Import.isabelle_tptp_file @{theory} 50 + "$TPTP/Problems/PUZ/PUZ107^5.p" *} *) end