src/HOL/Groups_Big.thy
changeset 66089 def95e0bc529
parent 65687 a68973661472
child 66112 0e640e04fc56
equal deleted inserted replaced
66088:c9c9438cfc0f 66089:def95e0bc529
   330   show ?thesis
   330   show ?thesis
   331     unfolding F_eq using fin nn eq
   331     unfolding F_eq using fin nn eq
   332     by (intro reindex_bij_betw_not_neutral[OF _ _ bij]) auto
   332     by (intro reindex_bij_betw_not_neutral[OF _ _ bij]) auto
   333 qed
   333 qed
   334 
   334 
   335 lemma delta:
   335 lemma delta [simp]:
   336   assumes fS: "finite S"
   336   assumes fS: "finite S"
   337   shows "F (\<lambda>k. if k = a then b k else \<^bold>1) S = (if a \<in> S then b a else \<^bold>1)"
   337   shows "F (\<lambda>k. if k = a then b k else \<^bold>1) S = (if a \<in> S then b a else \<^bold>1)"
   338 proof -
   338 proof -
   339   let ?f = "(\<lambda>k. if k = a then b k else \<^bold>1)"
   339   let ?f = "(\<lambda>k. if k = a then b k else \<^bold>1)"
   340   show ?thesis
   340   show ?thesis
   353       using union_disjoint [OF fAB dj, of ?f, unfolded eq [symmetric]] by simp
   353       using union_disjoint [OF fAB dj, of ?f, unfolded eq [symmetric]] by simp
   354     with True show ?thesis by simp
   354     with True show ?thesis by simp
   355   qed
   355   qed
   356 qed
   356 qed
   357 
   357 
   358 lemma delta':
   358 lemma delta' [simp]:
   359   assumes fin: "finite S"
   359   assumes fin: "finite S"
   360   shows "F (\<lambda>k. if a = k then b k else \<^bold>1) S = (if a \<in> S then b a else \<^bold>1)"
   360   shows "F (\<lambda>k. if a = k then b k else \<^bold>1) S = (if a \<in> S then b a else \<^bold>1)"
   361   using delta [OF fin, of a b, symmetric] by (auto intro: cong)
   361   using delta [OF fin, of a b, symmetric] by (auto intro: cong)
   362 
   362 
   363 lemma If_cases:
   363 lemma If_cases: