src/ZF/Perm.thy
changeset 63901 4ce989e962e0
parent 60770 240563fbf41d
child 67399 eab6ce8368fa
--- a/src/ZF/Perm.thy	Fri Sep 16 18:09:13 2016 +0200
+++ b/src/ZF/Perm.thy	Fri Sep 16 21:28:09 2016 +0200
@@ -137,7 +137,7 @@
 apply (blast intro!: lam_injective lam_surjective)
 done
 
-lemma RepFun_bijective: "(\<forall>y\<in>x. EX! y'. f(y') = f(y))
+lemma RepFun_bijective: "(\<forall>y\<in>x. \<exists>!y'. f(y') = f(y))
       ==> (\<lambda>z\<in>{f(y). y \<in> x}. THE y. f(y) = z) \<in> bij({f(y). y \<in> x}, x)"
 apply (rule_tac d = f in lam_bijective)
 apply (auto simp add: the_equality2)