src/HOL/BNF/BNF_FP.thy
changeset 49585 5c4a12550491
parent 49539 be6cbf960aa7
child 49590 43e2d0e10876
--- a/src/HOL/BNF/BNF_FP.thy	Wed Sep 26 10:00:59 2012 +0200
+++ b/src/HOL/BNF/BNF_FP.thy	Wed Sep 26 10:00:59 2012 +0200
@@ -14,6 +14,9 @@
   "defaults"
 begin
 
+lemma eq_sym_Unity_imp: "x = (() = ()) \<Longrightarrow> x"
+by blast
+
 lemma unit_case_Unity: "(case u of () => f) = f"
 by (cases u) (hypsubst, rule unit.cases)
 
@@ -97,6 +100,11 @@
 lemma mem_UN_compreh_eq: "(z : \<Union>{y. \<exists>x\<in>A. y = F x}) = (\<exists>x\<in>A. z : F x)"
 by blast
 
+lemma UN_compreh_eq_eq:
+"\<Union>{y. \<exists>x\<in>A. y = {}} = {}"
+"\<Union>{y. \<exists>x\<in>A. y = {x}} = A"
+by blast+
+
 lemma prod_set_simps:
 "fsts (x, y) = {x}"
 "snds (x, y) = {y}"