src/HOL/TPTP/TPTP_Test.thy
changeset 47547 1a5dc8377b5c
parent 47518 b2f209258621
child 47558 55b42f9af99d
--- a/src/HOL/TPTP/TPTP_Test.thy	Wed Apr 18 18:24:16 2012 +0200
+++ b/src/HOL/TPTP/TPTP_Test.thy	Wed Apr 18 17:33:11 2012 +0100
@@ -102,6 +102,7 @@
 
 ML {*
   fun situate file_name = Path.append tptp_probs_dir (Path.explode file_name);
+
   fun parser_test ctxt = (*FIXME argument order*)
     test_fn ctxt
      (fn file_name =>
@@ -111,6 +112,9 @@
               TPTP_Parser.parse_file file)))
      "parser"
      ()
+
+  fun parse_timed file =
+    Timing.timing TPTP_Parser.parse_file (Path.implode file)
 *}
 
 end
\ No newline at end of file