equal
deleted
inserted
replaced
584 "integral\<^sup>S M f = (\<Sum>x \<in> f ` space M. x * emeasure M (f -` {x} \<inter> space M))" |
584 "integral\<^sup>S M f = (\<Sum>x \<in> f ` space M. x * emeasure M (f -` {x} \<inter> space M))" |
585 |
585 |
586 syntax |
586 syntax |
587 "_simple_integral" :: "pttrn \<Rightarrow> ennreal \<Rightarrow> 'a measure \<Rightarrow> ennreal" ("\<integral>\<^sup>S _. _ \<partial>_" [60,61] 110) |
587 "_simple_integral" :: "pttrn \<Rightarrow> ennreal \<Rightarrow> 'a measure \<Rightarrow> ennreal" ("\<integral>\<^sup>S _. _ \<partial>_" [60,61] 110) |
588 |
588 |
|
589 syntax_consts |
|
590 "_simple_integral" == simple_integral |
|
591 |
589 translations |
592 translations |
590 "\<integral>\<^sup>S x. f \<partial>M" == "CONST simple_integral M (%x. f)" |
593 "\<integral>\<^sup>S x. f \<partial>M" == "CONST simple_integral M (%x. f)" |
591 |
594 |
592 lemma simple_integral_cong: |
595 lemma simple_integral_cong: |
593 assumes "\<And>t. t \<in> space M \<Longrightarrow> f t = g t" |
596 assumes "\<And>t. t \<in> space M \<Longrightarrow> f t = g t" |
816 definition\<^marker>\<open>tag important\<close> nn_integral :: "'a measure \<Rightarrow> ('a \<Rightarrow> ennreal) \<Rightarrow> ennreal" ("integral\<^sup>N") where |
819 definition\<^marker>\<open>tag important\<close> nn_integral :: "'a measure \<Rightarrow> ('a \<Rightarrow> ennreal) \<Rightarrow> ennreal" ("integral\<^sup>N") where |
817 "integral\<^sup>N M f = (SUP g \<in> {g. simple_function M g \<and> g \<le> f}. integral\<^sup>S M g)" |
820 "integral\<^sup>N M f = (SUP g \<in> {g. simple_function M g \<and> g \<le> f}. integral\<^sup>S M g)" |
818 |
821 |
819 syntax |
822 syntax |
820 "_nn_integral" :: "pttrn \<Rightarrow> ennreal \<Rightarrow> 'a measure \<Rightarrow> ennreal" ("\<integral>\<^sup>+((2 _./ _)/ \<partial>_)" [60,61] 110) |
823 "_nn_integral" :: "pttrn \<Rightarrow> ennreal \<Rightarrow> 'a measure \<Rightarrow> ennreal" ("\<integral>\<^sup>+((2 _./ _)/ \<partial>_)" [60,61] 110) |
|
824 |
|
825 syntax_consts |
|
826 "_nn_integral" == nn_integral |
821 |
827 |
822 translations |
828 translations |
823 "\<integral>\<^sup>+x. f \<partial>M" == "CONST nn_integral M (\<lambda>x. f)" |
829 "\<integral>\<^sup>+x. f \<partial>M" == "CONST nn_integral M (\<lambda>x. f)" |
824 |
830 |
825 lemma nn_integral_def_finite: |
831 lemma nn_integral_def_finite: |