src/HOL/TPTP/TPTP_Interpret_Test.thy
changeset 58412 f65f11f4854c
parent 56303 4cc3f4db3447
child 62390 842917225d56
--- a/src/HOL/TPTP/TPTP_Interpret_Test.thy	Sun Sep 21 19:53:50 2014 +0200
+++ b/src/HOL/TPTP/TPTP_Interpret_Test.thy	Sun Sep 21 20:14:04 2014 +0200
@@ -55,7 +55,7 @@
   fun interpretation_tests timeout ctxt probs =
     List.app
      (interpretation_test timeout ctxt)
-     (List.map situate probs)
+     (map situate probs)
 *}
 
 ML {*