src/HOL/Library/FuncSet.thy
changeset 70063 adaa0a6ea4fe
parent 69939 812ce526da33
child 71258 d67924987c34
--- a/src/HOL/Library/FuncSet.thy	Thu Apr 04 16:38:45 2019 +0100
+++ b/src/HOL/Library/FuncSet.thy	Fri Apr 05 11:21:53 2019 +0100
@@ -220,6 +220,12 @@
 lemma restrict_Pi_cancel: "restrict x I \<in> Pi I A \<longleftrightarrow> x \<in> Pi I A"
   by (auto simp: restrict_def Pi_def)
 
+lemma sum_restrict' [simp]: "sum' (\<lambda>i\<in>I. g i) I = sum' (\<lambda>i. g i) I"
+  by (simp add: sum.G_def conj_commute cong: conj_cong)
+
+lemma prod_restrict' [simp]: "prod' (\<lambda>i\<in>I. g i) I = prod' (\<lambda>i. g i) I"
+  by (simp add: prod.G_def conj_commute cong: conj_cong)
+
 
 subsection \<open>Bijections Between Sets\<close>