| author | wenzelm | 
| Mon, 15 Jul 2013 10:42:12 +0200 | |
| changeset 52657 | 42c14dba1daa | 
| parent 52487 | 48bc24467008 | 
| child 57812 | 8dc9dc241973 | 
| permissions | -rw-r--r-- | 
| 46324 | 1 | (* Title: HOL/TPTP/ATP_Problem_Import.thy | 
| 2 | Author: Jasmin Blanchette, TU Muenchen | |
| 3 | *) | |
| 4 | ||
| 5 | header {* ATP Problem Importer *}
 | |
| 47812 | 6 | |
| 46324 | 7 | theory ATP_Problem_Import | 
| 49985 
5b4b0e4e5205
moved Refute to "HOL/Library" to speed up building "Main" even more
 blanchet parents: 
48891diff
changeset | 8 | imports | 
| 
5b4b0e4e5205
moved Refute to "HOL/Library" to speed up building "Main" even more
 blanchet parents: 
48891diff
changeset | 9 | Complex_Main | 
| 
5b4b0e4e5205
moved Refute to "HOL/Library" to speed up building "Main" even more
 blanchet parents: 
48891diff
changeset | 10 | TPTP_Interpret | 
| 
5b4b0e4e5205
moved Refute to "HOL/Library" to speed up building "Main" even more
 blanchet parents: 
48891diff
changeset | 11 | "~~/src/HOL/Library/Refute" | 
| 46324 | 12 | begin | 
| 13 | ||
| 48891 | 14 | ML_file "sledgehammer_tactics.ML" | 
| 15 | ||
| 52487 
48bc24467008
backout dedd7952a62c: static "proofs" value within theory prevents later inferencing with different configuration;
 wenzelm parents: 
52470diff
changeset | 16 | ML {* Proofterm.proofs := 0 *}
 | 
| 47765 | 17 | |
| 47670 | 18 | declare [[show_consts]] (* for Refute *) | 
| 47765 | 19 | declare [[smt_oracle]] | 
| 47670 | 20 | |
| 47794 
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
 blanchet parents: 
47790diff
changeset | 21 | declare [[unify_search_bound = 60]] | 
| 
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
 blanchet parents: 
47790diff
changeset | 22 | declare [[unify_trace_bound = 60]] | 
| 
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
 blanchet parents: 
47790diff
changeset | 23 | |
| 48891 | 24 | ML_file "atp_problem_import.ML" | 
| 47794 
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
 blanchet parents: 
47790diff
changeset | 25 | |
| 47785 | 26 | (* | 
| 47794 
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
 blanchet parents: 
47790diff
changeset | 27 | ML {* ATP_Problem_Import.isabelle_tptp_file @{theory} 50
 | 
| 
4ad62c5f9f88
thread theory cleanly and use "smt" method rather than Sledgehammer for Z3 (because of obscure debilitating bug)
 blanchet parents: 
47790diff
changeset | 28 | "$TPTP/Problems/PUZ/PUZ107^5.p" *} | 
| 47785 | 29 | *) | 
| 30 | ||
| 46324 | 31 | end |