src/HOL/Set.thy
changeset 69144 f13b82281715
parent 68780 54fdc8bc73a3
child 69163 6c9453ec2191
--- a/src/HOL/Set.thy	Wed Oct 17 07:50:46 2018 +0200
+++ b/src/HOL/Set.thy	Wed Oct 17 14:19:07 2018 +0100
@@ -1140,6 +1140,8 @@
 lemma not_psubset_empty [iff]: "\<not> (A < {})"
   by (fact not_less_bot) (* FIXME: already simp *)
 
+lemma Collect_subset [simp]: "{x\<in>A. P x} \<subseteq> A" by auto
+
 lemma Collect_empty_eq [simp]: "Collect P = {} \<longleftrightarrow> (\<forall>x. \<not> P x)"
   by blast