src/HOL/Nitpick_Examples/Mono_Nits.thy
changeset 59058 a78612c67ec0
parent 58889 5b7a9633cfa8
child 59582 0fbed69ff081
--- a/src/HOL/Nitpick_Examples/Mono_Nits.thy	Wed Nov 26 16:55:43 2014 +0100
+++ b/src/HOL/Nitpick_Examples/Mono_Nits.thy	Wed Nov 26 20:05:34 2014 +0100
@@ -153,7 +153,7 @@
 fun theorems_of thy =
   filter (fn (name, th) =>
              not (is_forbidden_theorem name) andalso
-             (theory_of_thm th, thy) |> pairself Context.theory_name |> op =)
+             (theory_of_thm th, thy) |> apply2 Context.theory_name |> op =)
          (Global_Theory.all_thms_of thy true)
 
 fun check_formulas tsp =