src/HOL/TPTP/TPTP_Interpret_Test.thy
changeset 55595 2e2e9bc7c4c6
parent 48829 6ed588c4f963
child 56303 4cc3f4db3447
--- a/src/HOL/TPTP/TPTP_Interpret_Test.thy	Wed Feb 19 15:57:02 2014 +0000
+++ b/src/HOL/TPTP/TPTP_Interpret_Test.thy	Wed Feb 19 15:57:02 2014 +0000
@@ -154,7 +154,7 @@
 ML {*
   if test_all @{context} then
     (report @{context} "Interpreting all problems";
-     S timed_test (interpretation_test (get_timeout @{context})) @{context})
+     S timed_test (interpretation_test (get_timeout @{context})) @{context} (TPTP_Syntax.get_file_list tptp_probs_dir))
   else ()
 *}