]> matita.cs.unibo.it Git - helm.git/commitdiff
more properties of union
authorAndrea Asperti <andrea.asperti@unibo.it>
Tue, 3 Jan 2012 15:57:18 +0000 (15:57 +0000)
committerAndrea Asperti <andrea.asperti@unibo.it>
Tue, 3 Jan 2012 15:57:18 +0000 (15:57 +0000)
matita/matita/lib/basics/sets.ma

index bb077e65384db670bc10bb4fe184cf8c92ee6d46..4d77f6c2f86f5808bbdbe6e416ca6676969e6f86 100644 (file)
@@ -74,6 +74,11 @@ lemma eqP_substract_l: ∀U.∀A,B,C:U →Prop.
 #U #A #B #C #eqBC #a @iff_and_l /2/ qed.
 
 (* set equalities *)
+lemma union_empty_r: ∀U.∀A:U→Prop. 
+  A ∪ ∅ =1 A.
+#U #A #w % [* // normalize #abs @False_ind /2/ | /2/]
+qed.
+
 lemma union_comm : ∀U.∀A,B:U →Prop. 
   A ∪ B =1 B ∪ A.
 #U #A #B #a % * /2/ qed.