src/HOL/Library/Indicator_Function.thy
changeset 63092 a949b2a5f51d
parent 62648 ee48e0b4f669
child 63099 af0e964aad7b
--- a/src/HOL/Library/Indicator_Function.thy	Fri May 13 20:22:02 2016 +0200
+++ b/src/HOL/Library/Indicator_Function.thy	Fri May 13 20:24:10 2016 +0200
@@ -79,7 +79,7 @@
 lemma setsum_indicator_scaleR[simp]:
   "finite A \<Longrightarrow>
     (\<Sum>x \<in> A. indicator (B x) (g x) *\<^sub>R f x) = (\<Sum>x \<in> {x\<in>A. g x \<in> B x}. f x::'a::real_vector)"
-  using assms by (auto intro!: setsum.mono_neutral_cong_right split: if_split_asm simp: indicator_def)
+  by (auto intro!: setsum.mono_neutral_cong_right split: if_split_asm simp: indicator_def)
 
 lemma LIMSEQ_indicator_incseq:
   assumes "incseq A"