diff -r f13a762f7d96 -r 1557a391a858 src/HOL/Set.thy --- 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 \ B \ A \ f -` B" + by blast + lemma vimage_const [simp]: "((\x. c) -` A) = (if c \ A then UNIV else {})" by auto