src/HOL/TPTP/TPTP_Interpret_Test.thy
changeset 48829 6ed588c4f963
parent 47693 64023cf4d148
child 55595 2e2e9bc7c4c6
--- a/src/HOL/TPTP/TPTP_Interpret_Test.thy	Thu Aug 16 14:07:32 2012 +0200
+++ b/src/HOL/TPTP/TPTP_Interpret_Test.thy	Thu Aug 16 15:41:36 2012 +0200
@@ -17,7 +17,7 @@
     Timing.timing
       (TPTP_Interpret.interpret_file
        false
-       (Path.dir tptp_probs_dir)
+       [Path.explode "$TPTP"]
        (Path.append tptp_probs_dir (Path.explode "LCL/LCL825-1.p"))
        []
        [])
@@ -38,7 +38,7 @@
     TimeLimit.timeLimit (Time.fromSeconds (if timeout = 0 then 60 else timeout))
      (TPTP_Interpret.interpret_file
        false
-       (Path.dir tptp_probs_dir)
+       [Path.explode "$TPTP"]
        file
        []
        []) thy