src/ZF/AC.thy
changeset 76215 a642599ffdea
parent 76213 e44d86131648
--- a/src/ZF/AC.thy	Tue Sep 27 17:03:23 2022 +0100
+++ b/src/ZF/AC.thy	Tue Sep 27 17:46:52 2022 +0100
@@ -26,13 +26,13 @@
 done
 
 lemma AC_Pi_Pow: "\<exists>f. f \<in> (\<Prod>X \<in> Pow(C)-{0}. X)"
-apply (rule_tac B1 = "%x. x" in AC_Pi [THEN exE])
+apply (rule_tac B1 = "\<lambda>x. x" in AC_Pi [THEN exE])
 apply (erule_tac [2] exI, blast)
 done
 
 lemma AC_func:
      "\<lbrakk>\<And>x. x \<in> A \<Longrightarrow> (\<exists>y. y \<in> x)\<rbrakk> \<Longrightarrow> \<exists>f \<in> A->\<Union>(A). \<forall>x \<in> A. f`x \<in> x"
-apply (rule_tac B1 = "%x. x" in AC_Pi [THEN exE])
+apply (rule_tac B1 = "\<lambda>x. x" in AC_Pi [THEN exE])
 prefer 2 apply (blast dest: apply_type intro: Pi_type, blast)
 done