diff -r 26c501c5024d -r 8bad1f42fec0 src/HOL/Reconstruction.thy --- a/src/HOL/Reconstruction.thy Thu Dec 02 10:36:20 2004 +0100 +++ b/src/HOL/Reconstruction.thy Thu Dec 02 11:09:19 2004 +0100 @@ -8,7 +8,13 @@ theory Reconstruction imports Hilbert_Choice - files "Tools/reconstruction.ML" + 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