src/HOL/Analysis/Henstock_Kurzweil_Integration.thy
changeset 73536 5131c388a9b0
parent 73373 3bb9df8900fd
child 73928 3b76524f5a85
child 73932 fd21b4a93043
equal deleted inserted replaced
73535:0f33c7031ec9 73536:5131c388a9b0
  2334   have "(indicat_real (S \<union> T) has_integral 0) (cbox a b)"
  2334   have "(indicat_real (S \<union> T) has_integral 0) (cbox a b)"
  2335     if S0: "(indicat_real S has_integral 0) (cbox a b)" 
  2335     if S0: "(indicat_real S has_integral 0) (cbox a b)" 
  2336       and  "(indicat_real T has_integral 0) (cbox a b)" for a b
  2336       and  "(indicat_real T has_integral 0) (cbox a b)" for a b
  2337   proof (subst has_integral_spike_eq[OF T])
  2337   proof (subst has_integral_spike_eq[OF T])
  2338     show "indicat_real S x = indicat_real (S \<union> T) x" if "x \<in> cbox a b - T" for x
  2338     show "indicat_real S x = indicat_real (S \<union> T) x" if "x \<in> cbox a b - T" for x
  2339       by (metis Diff_iff Un_iff indicator_def that)
  2339       using that by (simp add: indicator_def)
  2340     show "(indicat_real S has_integral 0) (cbox a b)"
  2340     show "(indicat_real S has_integral 0) (cbox a b)"
  2341       by (simp add: S0)
  2341       by (simp add: S0)
  2342   qed
  2342   qed
  2343   with assms show ?thesis
  2343   with assms show ?thesis
  2344     unfolding negligible_def by blast
  2344     unfolding negligible_def by blast