src/HOL/Reconstruction.thy
author paulson
Fri, 20 Aug 2004 12:21:03 +0200
changeset 15151 429666b09783
child 15359 8bad1f42fec0
permissions -rw-r--r--
proof reconstruction for external ATPs
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
15151
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
     1
(*  Title:      HOL/Reconstruction.thy
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
     2
    ID: $Id$
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
     3
    Author:     Lawrence C Paulson
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
     4
    Copyright   2004  University of Cambridge
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
     5
*)
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
     6
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
     7
header{*Attributes for Reconstructing External Resolution Proofs*}
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
     8
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
     9
theory Reconstruction
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
    10
    imports Hilbert_Choice
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
    11
    files   "Tools/reconstruction.ML"
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
    12
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
    13
begin
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
    14
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
    15
setup Reconstruction.setup
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
    16
429666b09783 proof reconstruction for external ATPs
paulson
parents:
diff changeset
    17
end