src/HOL/UNITY/PPROD.thy
changeset 67613 ce654b0e6d69
parent 63146 f1ecba0272f9
child 69597 ff784d5a5bfb
--- a/src/HOL/UNITY/PPROD.thy	Tue Feb 13 14:24:50 2018 +0100
+++ b/src/HOL/UNITY/PPROD.thy	Thu Feb 15 12:11:00 2018 +0100
@@ -120,8 +120,8 @@
   something like \<open>lift_preserves_sub\<close> to rewrite the third.  However
   there's no obvious alternative for the third premise.\<close>
 lemma guarantees_PLam_I:
-    "[| lift i (F i): X guarantees Y;  i \<in> I;
-        OK I (%i. lift i (F i)) |]
+    "[| lift i (F i) \<in> X guarantees Y;  i \<in> I;
+        OK I (\<lambda>i. lift i (F i)) |]
      ==> (PLam I F) \<in> X guarantees Y"
 apply (unfold PLam_def)
 apply (simp add: guarantees_JN_I)