--- a/src/Tools/Compute_Oracle/Compute_Oracle.thy Sat Oct 27 18:37:06 2007 +0200
+++ b/src/Tools/Compute_Oracle/Compute_Oracle.thy Sat Oct 27 18:37:32 2007 +0200
@@ -6,9 +6,9 @@
*)
theory Compute_Oracle imports CPure
-uses "am.ML" "am_compiler.ML" "am_interpreter.ML" "am_ghc.ML" "am_sml.ML" "compute.ML" "linker.ML"
+uses "am.ML" "am_compiler.ML" "am_interpreter.ML" "am_ghc.ML" "am_sml.ML" "report.ML" "compute.ML" "linker.ML"
begin
-setup {* Compute.setup; *}
+setup {* Compute.setup_compute; *}
end
\ No newline at end of file