src/HOL/Analysis/Henstock_Kurzweil_Integration.thy
changeset 73536 5131c388a9b0
parent 73373 3bb9df8900fd
child 73928 3b76524f5a85
child 73932 fd21b4a93043
--- a/src/HOL/Analysis/Henstock_Kurzweil_Integration.thy	Tue Apr 06 18:12:20 2021 +0000
+++ b/src/HOL/Analysis/Henstock_Kurzweil_Integration.thy	Wed Apr 07 12:28:19 2021 +0000
@@ -2336,7 +2336,7 @@
       and  "(indicat_real T has_integral 0) (cbox a b)" for a b
   proof (subst has_integral_spike_eq[OF T])
     show "indicat_real S x = indicat_real (S \<union> T) x" if "x \<in> cbox a b - T" for x
-      by (metis Diff_iff Un_iff indicator_def that)
+      using that by (simp add: indicator_def)
     show "(indicat_real S has_integral 0) (cbox a b)"
       by (simp add: S0)
   qed