src/HOL/Analysis/Henstock_Kurzweil_Integration.thy
changeset 69517 dc20f278e8f3
parent 69510 0f31dd2e540d
child 69529 4ab9657b3257
--- a/src/HOL/Analysis/Henstock_Kurzweil_Integration.thy	Thu Dec 27 23:38:55 2018 +0100
+++ b/src/HOL/Analysis/Henstock_Kurzweil_Integration.thy	Fri Dec 28 10:29:59 2018 +0100
@@ -3,11 +3,12 @@
                 Huge cleanup by LCP
 *)
 
-section \<open>Henstock-Kurzweil gauge integration in many dimensions\<close>
+section \<open>Henstock-Kurzweil Gauge Integration in Many Dimensions\<close>
 
 theory Henstock_Kurzweil_Integration
 imports
-  Lebesgue_Measure Tagged_Division
+  Lebesgue_Measure
+  Tagged_Division
 begin
 
 lemma norm_diff2: "\<lbrakk>y = y1 + y2; x = x1 + x2; e = e1 + e2; norm(y1 - x1) \<le> e1; norm(y2 - x2) \<le> e2\<rbrakk>