src/HOL/TPTP/TPTP_Parser_Test.thy
changeset 69366 b6dacf6eabe3
parent 68672 9247996782c9
--- a/src/HOL/TPTP/TPTP_Parser_Test.thy	Wed Nov 28 15:38:18 2018 +0100
+++ b/src/HOL/TPTP/TPTP_Parser_Test.thy	Wed Nov 28 16:14:31 2018 +0100
@@ -47,7 +47,7 @@
 
 (*test against all TPTP problems*)
 fun problem_names () =
-    map (Path.base_name #>
+    map (Path.file_name #>
          TPTP_Problem_Name.parse_problem_name #>
          TPTP_Problem_Name.mangle_problem_name)
      (TPTP_Syntax.get_file_list tptp_probs_dir)