src/HOL/Reconstruction.thy
author berghofe
Mon, 24 Jan 2005 18:18:28 +0100
changeset 15464 02cc838b64ca
parent 15382 e56ce5cefe9c
child 15645 5e20c54683d3
permissions -rw-r--r--
Added variant of eres_inst_tac that operates on indexnames instead of strings.

(*  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 Map Infinite_Set
    files "Tools/res_lib.ML"
	  "Tools/res_clause.ML"
	  "Tools/res_skolem_function.ML"
	  "Tools/res_axioms.ML"
	  "Tools/res_types_sorts.ML"
	  "Tools/res_atp.ML"
          "Tools/reconstruction.ML"

begin

text{*Every theory of HOL must be a descendant or ancestor of this one!*}

setup Reconstruction.setup

end