src/ZF/Perm.thy
changeset 47101 ded5cc757bc9
parent 46953 2b6e55924af3
child 58871 c399ae4b836f
--- a/src/ZF/Perm.thy	Fri Mar 23 12:03:59 2012 +0100
+++ b/src/ZF/Perm.thy	Fri Mar 23 16:16:15 2012 +0000
@@ -505,6 +505,9 @@
 apply (blast intro: apply_equality apply_Pair Pi_type)
 done
 
+lemma surj_image_eq: "f \<in> surj(A, B) ==> f``A = B"
+  by (auto simp add: surj_def image_fun) (blast dest: apply_type) 
+
 lemma restrict_image [simp]: "restrict(f,A) `` B = f `` (A \<inter> B)"
 by (auto simp add: restrict_def)