src/HOL/Analysis/Bochner_Integration.thy
changeset 81182 fc5066122e68
parent 81097 6c81cdca5b82
--- a/src/HOL/Analysis/Bochner_Integration.thy	Fri Oct 18 11:44:05 2024 +0200
+++ b/src/HOL/Analysis/Bochner_Integration.thy	Fri Oct 18 14:20:09 2024 +0200
@@ -892,20 +892,16 @@
 syntax
   "_lebesgue_integral" :: "pttrn \<Rightarrow> real \<Rightarrow> 'a measure \<Rightarrow> real"
     (\<open>(\<open>indent=1 notation=\<open>binder integral\<close>\<close>\<integral>(2 _./ _)/ \<partial>_)\<close> [60,61] 110)
-
 syntax_consts
   "_lebesgue_integral" == lebesgue_integral
-
 translations
   "\<integral> x. f \<partial>M" == "CONST lebesgue_integral M (\<lambda>x. f)"
 
 syntax
   "_ascii_lebesgue_integral" :: "pttrn \<Rightarrow> 'a measure \<Rightarrow> real \<Rightarrow> real"
     (\<open>(\<open>indent=3 notation=\<open>mixfix LINT\<close>\<close>LINT (1_)/|(_)./ _)\<close> [0,110,60] 60)
-
 syntax_consts
   "_ascii_lebesgue_integral" == lebesgue_integral
-
 translations
   "LINT x|M. f" == "CONST lebesgue_integral M (\<lambda>x. f)"