lemma Compl_insert: "- insert x A = (-A) - {x}"
authorkrauss
Thu, 25 Aug 2011 14:06:34 +0200
changeset 44490 e3e8d20a6ebc
parent 44489 6cddca146ca0
child 44491 ba22ed224b20
lemma Compl_insert: "- insert x A = (-A) - {x}"
src/HOL/Set.thy
--- a/src/HOL/Set.thy	Thu Aug 25 11:15:31 2011 +0200
+++ b/src/HOL/Set.thy	Thu Aug 25 14:06:34 2011 +0200
@@ -1378,6 +1378,9 @@
 lemma Compl_eq_Compl_iff [iff]: "(-A = -B) = (A = (B::'a set))"
   by (fact compl_eq_compl_iff)
 
+lemma Compl_insert: "- insert x A = (-A) - {x}"
+  by blast
+
 text {* \medskip Bounded quantifiers.
 
   The following are not added to the default simpset because