src/HOL/Predicate_Compile.thy
changeset 40052 ea46574ca815
parent 36046 c3946372f556
child 45450 dc2236b19a3d
--- a/src/HOL/Predicate_Compile.thy	Thu Oct 21 19:13:09 2010 +0200
+++ b/src/HOL/Predicate_Compile.thy	Thu Oct 21 19:13:09 2010 +0200
@@ -9,6 +9,9 @@
 uses
   "Tools/Predicate_Compile/predicate_compile_aux.ML"
   "Tools/Predicate_Compile/predicate_compile_compilations.ML"
+  "Tools/Predicate_Compile/core_data.ML"
+  "Tools/Predicate_Compile/mode_inference.ML"
+  "Tools/Predicate_Compile/predicate_compile_proof.ML"
   "Tools/Predicate_Compile/predicate_compile_core.ML"
   "Tools/Predicate_Compile/predicate_compile_data.ML"
   "Tools/Predicate_Compile/predicate_compile_fun.ML"