| author | wenzelm | 
| Tue, 08 Nov 2005 10:43:08 +0100 | |
| changeset 18117 | 61a430a67d7c | 
| parent 18004 | 1883971957de | 
| child 18449 | e314fb38307d | 
| permissions | -rw-r--r-- | 
| 15151 | 1 | (* Title: HOL/Reconstruction.thy | 
| 17603 | 2 | ID: $Id$ | 
| 15151 | 3 | Author: Lawrence C Paulson | 
| 4 | Copyright 2004 University of Cambridge | |
| 5 | *) | |
| 6 | ||
| 17462 
47f7bddc3239
moved setup ResAxioms.clause_setup to Main.thy (it refers to all previous theories);
 wenzelm parents: 
17421diff
changeset | 7 | header{* Reconstructing external resolution proofs *}
 | 
| 15151 | 8 | |
| 9 | theory Reconstruction | |
| 17508 | 10 | imports Hilbert_Choice Map Infinite_Set Extraction | 
| 17819 | 11 | uses "Tools/res_clause.ML" | 
| 18004 
1883971957de
Added a new file res_hol_clause.ML to Reconstruction.thy. This file is used to translate HOL formulae into FOL clauses.
 mengj parents: 
17846diff
changeset | 12 | "Tools/res_hol_clause.ML" | 
| 17819 | 13 | "Tools/res_axioms.ML" | 
| 14 | "Tools/ATP/recon_order_clauses.ML" | |
| 15 | "Tools/ATP/recon_translate_proof.ML" | |
| 16 | "Tools/ATP/recon_parse.ML" | |
| 17 | "Tools/ATP/recon_transfer_proof.ML" | |
| 18 | "Tools/ATP/AtpCommunication.ML" | |
| 19 | "Tools/ATP/watcher.ML" | |
| 20 | "Tools/ATP/res_clasimpset.ML" | |
| 21 | "Tools/res_atp.ML" | |
| 22 | "Tools/reconstruction.ML" | |
| 15151 | 23 | |
| 24 | begin | |
| 25 | ||
| 16563 | 26 | setup ResAxioms.meson_method_setup | 
| 15151 | 27 | setup Reconstruction.setup | 
| 28 | ||
| 15653 | 29 | end |