| author | wenzelm | 
| Wed, 05 Dec 2012 18:07:32 +0100 | |
| changeset 50372 | 11c96cac860d | 
| parent 50264 | a9ec48b98734 | 
| child 50923 | 141d8f575f6f | 
| permissions | -rw-r--r-- | 
| 35827 | 1 | (* Title: HOL/Sledgehammer.thy | 
| 38027 | 2 | Author: Lawrence C. Paulson, Cambridge University Computer Laboratory | 
| 38028 | 3 | Author: Jia Meng, Cambridge University Computer Laboratory and NICTA | 
| 35865 | 4 | Author: Jasmin Blanchette, TU Muenchen | 
| 21254 
d53f76357f41
incorporated former theories Reconstruction and ResAtpMethods into ATP_Linkup;
 wenzelm parents: diff
changeset | 5 | *) | 
| 
d53f76357f41
incorporated former theories Reconstruction and ResAtpMethods into ATP_Linkup;
 wenzelm parents: diff
changeset | 6 | |
| 35827 | 7 | header {* Sledgehammer: Isabelle--ATP Linkup *}
 | 
| 21254 
d53f76357f41
incorporated former theories Reconstruction and ResAtpMethods into ATP_Linkup;
 wenzelm parents: diff
changeset | 8 | |
| 35827 | 9 | theory Sledgehammer | 
| 40181 | 10 | imports ATP SMT | 
| 46950 
d0181abdbdac
declare command keywords via theory header, including strict checking outside Pure;
 wenzelm parents: 
43085diff
changeset | 11 | keywords "sledgehammer" :: diag and "sledgehammer_params" :: thy_decl | 
| 21254 
d53f76357f41
incorporated former theories Reconstruction and ResAtpMethods into ATP_Linkup;
 wenzelm parents: diff
changeset | 12 | begin | 
| 
d53f76357f41
incorporated former theories Reconstruction and ResAtpMethods into ATP_Linkup;
 wenzelm parents: diff
changeset | 13 | |
| 48891 | 14 | ML_file "Tools/Sledgehammer/async_manager.ML" | 
| 15 | ML_file "Tools/Sledgehammer/sledgehammer_util.ML" | |
| 16 | ML_file "Tools/Sledgehammer/sledgehammer_fact.ML" | |
| 50264 
a9ec48b98734
renamed sledgehammer_isar_reconstruct to sledgehammer_proof
 smolkas parents: 
50259diff
changeset | 17 | ML_file "Tools/Sledgehammer/sledgehammer_proof.ML" | 
| 50258 | 18 | ML_file "Tools/Sledgehammer/sledgehammer_annotate.ML" | 
| 50259 | 19 | ML_file "Tools/Sledgehammer/sledgehammer_shrink.ML" | 
| 49881 
d9d73ebf9274
added proof minimization code from Steffen Smolka
 blanchet parents: 
48891diff
changeset | 20 | ML_file "Tools/Sledgehammer/sledgehammer_reconstruct.ML" | 
| 48891 | 21 | ML_file "Tools/Sledgehammer/sledgehammer_provers.ML" | 
| 22 | ML_file "Tools/Sledgehammer/sledgehammer_minimize.ML" | |
| 23 | ML_file "Tools/Sledgehammer/sledgehammer_mepo.ML" | |
| 24 | ML_file "Tools/Sledgehammer/sledgehammer_mash.ML" | |
| 25 | ML_file "Tools/Sledgehammer/sledgehammer_run.ML" | |
| 26 | ML_file "Tools/Sledgehammer/sledgehammer_isar.ML" | |
| 27 | ||
| 42616 
92715b528e78
added Attrib.setup_config_XXX conveniences, with implicit setup of the background theory;
 wenzelm parents: 
41094diff
changeset | 28 | setup {* Sledgehammer_Isar.setup *}
 | 
| 23444 | 29 | |
| 21254 
d53f76357f41
incorporated former theories Reconstruction and ResAtpMethods into ATP_Linkup;
 wenzelm parents: diff
changeset | 30 | end |