src/HOL/Analysis/Lebesgue_Measure.thy
changeset 67968 a5ad4c015d1c
parent 67673 c8caefb20564
child 67982 7643b005b29a
--- a/src/HOL/Analysis/Lebesgue_Measure.thy	Sun Apr 08 12:31:08 2018 +0200
+++ b/src/HOL/Analysis/Lebesgue_Measure.thy	Mon Apr 09 16:20:23 2018 +0200
@@ -978,7 +978,8 @@
   then show ?thesis
     by (auto dest!: AE_not_in)
 qed
-subsection\<open> A nice lemma for negligibility proofs.\<close>
+
+subsection \<open>A nice lemma for negligibility proofs\<close>
 
 lemma summable_iff_suminf_neq_top: "(\<And>n. f n \<ge> 0) \<Longrightarrow> \<not> summable f \<Longrightarrow> (\<Sum>i. ennreal (f i)) = top"
   by (metis summable_suminf_not_top)