added lemmas rel_comp_UNION_distrib(2)
authorkrauss
Sun, 09 May 2010 12:00:43 +0200
changeset 36772 ef97c5006840
parent 36771 3e08b6789e66
child 36773 acb789f3936b
added lemmas rel_comp_UNION_distrib(2)
src/HOL/Relation.thy
--- a/src/HOL/Relation.thy	Sat May 08 22:29:44 2010 +0200
+++ b/src/HOL/Relation.thy	Sun May 09 12:00:43 2010 +0200
@@ -181,6 +181,12 @@
 lemma rel_comp_distrib2[simp]: "(S \<union> T) O R = (S O R) \<union> (T O R)"
 by auto
 
+lemma rel_comp_UNION_distrib: "s O UNION I r = UNION I (%i. s O r i)"
+by auto
+
+lemma rel_comp_UNION_distrib2: "UNION I r O s = UNION I (%i. r i O s)"
+by auto
+
 
 subsection {* Reflexivity *}