src/HOL/TPTP/TPTP_Interpret_Test.thy
changeset 55595 2e2e9bc7c4c6
parent 48829 6ed588c4f963
child 56303 4cc3f4db3447
equal deleted inserted replaced
55594:eb291b215c73 55595:2e2e9bc7c4c6
   152 text "Run interpretation over all problems. This works only for logics
   152 text "Run interpretation over all problems. This works only for logics
   153  for which interpretation is defined (in TPTP_Parser/tptp_interpret.ML)."
   153  for which interpretation is defined (in TPTP_Parser/tptp_interpret.ML)."
   154 ML {*
   154 ML {*
   155   if test_all @{context} then
   155   if test_all @{context} then
   156     (report @{context} "Interpreting all problems";
   156     (report @{context} "Interpreting all problems";
   157      S timed_test (interpretation_test (get_timeout @{context})) @{context})
   157      S timed_test (interpretation_test (get_timeout @{context})) @{context} (TPTP_Syntax.get_file_list tptp_probs_dir))
   158   else ()
   158   else ()
   159 *}
   159 *}
   160 
   160 
   161 end
   161 end