src/HOL/Set.thy
changeset 55775 1557a391a858
parent 55143 04448228381d
child 56014 aaa3f2365fc5
--- a/src/HOL/Set.thy	Thu Feb 27 15:19:09 2014 +0100
+++ b/src/HOL/Set.thy	Thu Feb 27 16:07:21 2014 +0000
@@ -1763,6 +1763,9 @@
 lemma image_vimage_eq [simp]: "f ` (f -` A) = A Int range f"
 by blast
 
+lemma image_subset_iff_subset_vimage: "f ` A \<subseteq> B \<longleftrightarrow> A \<subseteq> f -` B"
+  by blast 
+
 lemma vimage_const [simp]: "((\<lambda>x. c) -` A) = (if c \<in> A then UNIV else {})"
   by auto