| author | nipkow |
| Sat, 13 Nov 2004 07:47:34 +0100 | |
| changeset 15281 | bd4611956c7b |
| 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 |