| author | nipkow | 
| Mon, 22 Nov 2004 11:53:56 +0100 | |
| changeset 15305 | 0bd9eedaa301 | 
| parent 15151 | 429666b09783 | 
| child 15359 | 8bad1f42fec0 | 
| permissions | -rw-r--r-- | 
| 15151 | 1 | (* Title: HOL/Reconstruction.thy | 
| 2 | ID: $Id$ | |
| 3 | Author: Lawrence C Paulson | |
| 4 | Copyright 2004 University of Cambridge | |
| 5 | *) | |
| 6 | ||
| 7 | header{*Attributes for Reconstructing External Resolution Proofs*}
 | |
| 8 | ||
| 9 | theory Reconstruction | |
| 10 | imports Hilbert_Choice | |
| 11 | files "Tools/reconstruction.ML" | |
| 12 | ||
| 13 | begin | |
| 14 | ||
| 15 | setup Reconstruction.setup | |
| 16 | ||
| 17 | end |