src/HOL/Analysis/Nonnegative_Lebesgue_Integration.thy
changeset 81182 fc5066122e68
parent 81142 6ad2c917dd2e
--- a/src/HOL/Analysis/Nonnegative_Lebesgue_Integration.thy	Fri Oct 18 11:44:05 2024 +0200
+++ b/src/HOL/Analysis/Nonnegative_Lebesgue_Integration.thy	Fri Oct 18 14:20:09 2024 +0200
@@ -820,10 +820,8 @@
 
 syntax
   "_nn_integral" :: "pttrn \<Rightarrow> ennreal \<Rightarrow> 'a measure \<Rightarrow> ennreal" (\<open>(\<open>indent=2 notation=\<open>binder integral\<close>\<close>\<integral>\<^sup>+(2 _./ _)/ \<partial>_)\<close> [60,61] 110)
-
 syntax_consts
   "_nn_integral" == nn_integral
-
 translations
   "\<integral>\<^sup>+x. f \<partial>M" == "CONST nn_integral M (\<lambda>x. f)"