src/HOL/Reconstruction.thy
author aspinall
Fri, 01 Oct 2004 11:51:55 +0200
changeset 15220 cc88c8ee4d2f
parent 15151 429666b09783
child 15359 8bad1f42fec0
permissions -rw-r--r--
Comments

(*  Title:      HOL/Reconstruction.thy
    ID: $Id$
    Author:     Lawrence C Paulson
    Copyright   2004  University of Cambridge
*)

header{*Attributes for Reconstructing External Resolution Proofs*}

theory Reconstruction
    imports Hilbert_Choice
    files   "Tools/reconstruction.ML"

begin

setup Reconstruction.setup

end