src/HOL/Analysis/Infinite_Sum.thy
author wenzelm
Sun, 20 Oct 2024 21:48:38 +0200
changeset 81214 7c2745efec69
parent 81150 3dd8035578b8
child 82349 a854ca7ca7d9
permissions -rw-r--r--
clarified concrete vs. abstract syntax;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
     1
(*
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
     2
  Title:    HOL/Analysis/Infinite_Sum.thy
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
     3
  Author:   Dominique Unruh, University of Tartu
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
     4
            Manuel Eberl, University of Innsbruck
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
     5
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
     6
  A theory of sums over possibly infinite sets.
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
     7
*)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
     8
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
     9
section \<open>Infinite sums\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    10
\<^latex>\<open>\label{section:Infinite_Sum}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    11
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    12
text \<open>In this theory, we introduce the definition of infinite sums, i.e., sums ranging over an
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    13
infinite, potentially uncountable index set with no particular ordering.
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    14
(This is different from series. Those are sums indexed by natural numbers,
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    15
and the order of the index set matters.)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    16
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    17
Our definition is quite standard: $s:=\sum_{x\in A} f(x)$ is the limit of finite sums $s_F:=\sum_{x\in F} f(x)$ for increasing $F$.
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    18
That is, $s$ is the limit of the net $s_F$ where $F$ are finite subsets of $A$ ordered by inclusion.
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    19
We believe that this is the standard definition for such sums.
76987
4c275405faae isabelle update -u cite;
wenzelm
parents: 76940
diff changeset
    20
See, e.g., Definition 4.11 in \<^cite>\<open>"conway2013course"\<close>.
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    21
This definition is quite general: it is well-defined whenever $f$ takes values in some
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    22
commutative monoid endowed with a Hausdorff topology.
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    23
(Examples are reals, complex numbers, normed vector spaces, and more.)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    24
76999
ff203584b36e backed out changeset 7f7d5c93e36b: no longer required thanks to 9096703ed99e;
wenzelm
parents: 76988
diff changeset
    25
theory Infinite_Sum
ff203584b36e backed out changeset 7f7d5c93e36b: no longer required thanks to 9096703ed99e;
wenzelm
parents: 76988
diff changeset
    26
  imports
ff203584b36e backed out changeset 7f7d5c93e36b: no longer required thanks to 9096703ed99e;
wenzelm
parents: 76988
diff changeset
    27
    Elementary_Topology
ff203584b36e backed out changeset 7f7d5c93e36b: no longer required thanks to 9096703ed99e;
wenzelm
parents: 76988
diff changeset
    28
    "HOL-Library.Extended_Nonnegative_Real"
ff203584b36e backed out changeset 7f7d5c93e36b: no longer required thanks to 9096703ed99e;
wenzelm
parents: 76988
diff changeset
    29
    "HOL-Library.Complex_Order"
ff203584b36e backed out changeset 7f7d5c93e36b: no longer required thanks to 9096703ed99e;
wenzelm
parents: 76988
diff changeset
    30
begin
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    31
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    32
subsection \<open>Definition and syntax\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    33
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
    34
definition HAS_SUM :: \<open>('a \<Rightarrow> 'b :: {comm_monoid_add, topological_space}) \<Rightarrow> 'a set \<Rightarrow> 'b \<Rightarrow> bool\<close> 
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
    35
    where has_sum_def: \<open>HAS_SUM f A x \<equiv> (sum f \<longlongrightarrow> x) (finite_subsets_at_top A)\<close>
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
    36
80914
d97fdabd9e2b standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents: 80768
diff changeset
    37
abbreviation has_sum (infixr \<open>has'_sum\<close> 46) where
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
    38
  "(f has_sum S) A \<equiv> HAS_SUM f A S"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    39
80914
d97fdabd9e2b standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents: 80768
diff changeset
    40
definition summable_on :: "('a \<Rightarrow> 'b::{comm_monoid_add, topological_space}) \<Rightarrow> 'a set \<Rightarrow> bool" (infixr \<open>summable'_on\<close> 46) where
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
    41
  "f summable_on A \<equiv> (\<exists>x. (f has_sum x) A)"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    42
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    43
definition infsum :: "('a \<Rightarrow> 'b::{comm_monoid_add,t2_space}) \<Rightarrow> 'a set \<Rightarrow> 'b" where
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    44
  "infsum f A = (if f summable_on A then Lim (finite_subsets_at_top A) (sum f) else 0)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    45
80914
d97fdabd9e2b standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents: 80768
diff changeset
    46
abbreviation abs_summable_on :: "('a \<Rightarrow> 'b::real_normed_vector) \<Rightarrow> 'a set \<Rightarrow> bool" (infixr \<open>abs'_summable'_on\<close> 46) where
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    47
  "f abs_summable_on A \<equiv> (\<lambda>x. norm (f x)) summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    48
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    49
syntax (ASCII)
81097
6c81cdca5b82 more inner syntax markup: HOL-Analysis;
wenzelm
parents: 80914
diff changeset
    50
  "_infsum" :: "pttrn \<Rightarrow> 'a set \<Rightarrow> 'b \<Rightarrow> 'b::topological_comm_monoid_add"
6c81cdca5b82 more inner syntax markup: HOL-Analysis;
wenzelm
parents: 80914
diff changeset
    51
    (\<open>(\<open>indent=3 notation=\<open>binder INFSUM\<close>\<close>INFSUM (_/:_)./ _)\<close> [0, 51, 10] 10)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    52
syntax
81097
6c81cdca5b82 more inner syntax markup: HOL-Analysis;
wenzelm
parents: 80914
diff changeset
    53
  "_infsum" :: "pttrn \<Rightarrow> 'a set \<Rightarrow> 'b \<Rightarrow> 'b::topological_comm_monoid_add"
6c81cdca5b82 more inner syntax markup: HOL-Analysis;
wenzelm
parents: 80914
diff changeset
    54
    (\<open>(\<open>indent=2 notation=\<open>binder \<Sum>\<^sub>\<infinity>\<close>\<close>\<Sum>\<^sub>\<infinity>(_/\<in>_)./ _)\<close> [0, 51, 10] 10)
80768
c7723cc15de8 more markup for syntax consts;
wenzelm
parents: 79757
diff changeset
    55
syntax_consts
c7723cc15de8 more markup for syntax consts;
wenzelm
parents: 79757
diff changeset
    56
  "_infsum" \<rightleftharpoons> infsum
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    57
translations \<comment> \<open>Beware of argument permutation!\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    58
  "\<Sum>\<^sub>\<infinity>i\<in>A. b" \<rightleftharpoons> "CONST infsum (\<lambda>i. b) A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    59
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    60
syntax (ASCII)
81097
6c81cdca5b82 more inner syntax markup: HOL-Analysis;
wenzelm
parents: 80914
diff changeset
    61
  "_univinfsum" :: "pttrn \<Rightarrow> 'a \<Rightarrow> 'a"  (\<open>(\<open>indent=3 notation=\<open>binder INFSUM\<close>\<close>INFSUM _./ _)\<close> [0, 10] 10)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    62
syntax
81097
6c81cdca5b82 more inner syntax markup: HOL-Analysis;
wenzelm
parents: 80914
diff changeset
    63
  "_univinfsum" :: "pttrn \<Rightarrow> 'a \<Rightarrow> 'a"  (\<open>(\<open>indent=2 notation=\<open>binder \<Sum>\<^sub>\<infinity>\<close>\<close>\<Sum>\<^sub>\<infinity>_./ _)\<close> [0, 10] 10)
80768
c7723cc15de8 more markup for syntax consts;
wenzelm
parents: 79757
diff changeset
    64
syntax_consts
c7723cc15de8 more markup for syntax consts;
wenzelm
parents: 79757
diff changeset
    65
  "_univinfsum" \<rightleftharpoons> infsum
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    66
translations
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    67
  "\<Sum>\<^sub>\<infinity>x. t" \<rightleftharpoons> "CONST infsum (\<lambda>x. t) (CONST UNIV)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    68
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    69
syntax (ASCII)
81097
6c81cdca5b82 more inner syntax markup: HOL-Analysis;
wenzelm
parents: 80914
diff changeset
    70
  "_qinfsum" :: "pttrn \<Rightarrow> bool \<Rightarrow> 'a \<Rightarrow> 'a"  (\<open>(\<open>indent=3 notation=\<open>binder INFSUM\<close>\<close>INFSUM _ |/ _./ _)\<close> [0, 0, 10] 10)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    71
syntax
81097
6c81cdca5b82 more inner syntax markup: HOL-Analysis;
wenzelm
parents: 80914
diff changeset
    72
  "_qinfsum" :: "pttrn \<Rightarrow> bool \<Rightarrow> 'a \<Rightarrow> 'a"  (\<open>(\<open>indent=2 notation=\<open>binder \<Sum>\<^sub>\<infinity>\<close>\<close>\<Sum>\<^sub>\<infinity>_ | (_)./ _)\<close> [0, 0, 10] 10)
80768
c7723cc15de8 more markup for syntax consts;
wenzelm
parents: 79757
diff changeset
    73
syntax_consts
c7723cc15de8 more markup for syntax consts;
wenzelm
parents: 79757
diff changeset
    74
  "_qinfsum" \<rightleftharpoons> infsum
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    75
translations
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    76
  "\<Sum>\<^sub>\<infinity>x|P. t" => "CONST infsum (\<lambda>x. t) {x. P}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    77
print_translation \<open>
81150
3dd8035578b8 eliminate clones: just one Collect_binder_tr';
wenzelm
parents: 81097
diff changeset
    78
  [(\<^const_syntax>\<open>infsum\<close>, K (Collect_binder_tr' \<^syntax_const>\<open>_qinfsum\<close>))]
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    79
\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    80
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    81
subsection \<open>General properties\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    82
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    83
lemma infsumI:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    84
  fixes f g :: \<open>'a \<Rightarrow> 'b::{comm_monoid_add, t2_space}\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
    85
  assumes \<open>(f has_sum x) A\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    86
  shows \<open>infsum f A = x\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    87
  by (metis assms finite_subsets_at_top_neq_bot infsum_def summable_on_def has_sum_def tendsto_Lim)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    88
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    89
lemma infsum_eqI:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    90
  fixes f g :: \<open>'a \<Rightarrow> 'b::{comm_monoid_add, t2_space}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    91
  assumes \<open>x = y\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
    92
  assumes \<open>(f has_sum x) A\<close>
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
    93
  assumes \<open>(g has_sum y) B\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    94
  shows \<open>infsum f A = infsum g B\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
    95
  using assms infsumI by blast
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    96
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    97
lemma infsum_eqI':
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
    98
  fixes f g :: \<open>'a \<Rightarrow> 'b::{comm_monoid_add, t2_space}\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
    99
  assumes \<open>\<And>x. (f has_sum x) A \<longleftrightarrow> (g has_sum x) B\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   100
  shows \<open>infsum f A = infsum g B\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   101
  by (metis assms infsum_def infsum_eqI summable_on_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   102
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   103
lemma infsum_not_exists:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   104
  fixes f :: \<open>'a \<Rightarrow> 'b::{comm_monoid_add, t2_space}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   105
  assumes \<open>\<not> f summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   106
  shows \<open>infsum f A = 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   107
  by (simp add: assms infsum_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   108
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   109
lemma summable_iff_has_sum_infsum: "f summable_on A \<longleftrightarrow> (f has_sum (infsum f A)) A"
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   110
  using infsumI summable_on_def by blast
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   111
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   112
lemma has_sum_infsum[simp]:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   113
  assumes \<open>f summable_on S\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   114
  shows \<open>(f has_sum (infsum f S)) S\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   115
  using assms summable_iff_has_sum_infsum by blast
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   116
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   117
lemma has_sum_cong_neutral:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   118
  fixes f g :: \<open>'a \<Rightarrow> 'b::{comm_monoid_add, topological_space}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   119
  assumes \<open>\<And>x. x\<in>T-S \<Longrightarrow> g x = 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   120
  assumes \<open>\<And>x. x\<in>S-T \<Longrightarrow> f x = 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   121
  assumes \<open>\<And>x. x\<in>S\<inter>T \<Longrightarrow> f x = g x\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   122
  shows "(f has_sum x) S \<longleftrightarrow> (g has_sum x) T"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   123
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   124
  have \<open>eventually P (filtermap (sum f) (finite_subsets_at_top S))
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   125
      = eventually P (filtermap (sum g) (finite_subsets_at_top T))\<close> for P
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   126
  proof 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   127
    assume \<open>eventually P (filtermap (sum f) (finite_subsets_at_top S))\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   128
    then obtain F0 where \<open>finite F0\<close> and \<open>F0 \<subseteq> S\<close> and F0_P: \<open>\<And>F. finite F \<Longrightarrow> F \<subseteq> S \<Longrightarrow> F \<supseteq> F0 \<Longrightarrow> P (sum f F)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   129
      by (metis (no_types, lifting) eventually_filtermap eventually_finite_subsets_at_top)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   130
    define F0' where \<open>F0' = F0 \<inter> T\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   131
    have [simp]: \<open>finite F0'\<close> \<open>F0' \<subseteq> T\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   132
      by (simp_all add: F0'_def \<open>finite F0\<close>)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   133
    have \<open>P (sum g F)\<close> if \<open>finite F\<close> \<open>F \<subseteq> T\<close> \<open>F \<supseteq> F0'\<close> for F
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   134
    proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   135
      have \<open>P (sum f ((F\<inter>S) \<union> (F0\<inter>S)))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   136
        by (intro F0_P) (use \<open>F0 \<subseteq> S\<close> \<open>finite F0\<close> that in auto)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   137
      also have \<open>sum f ((F\<inter>S) \<union> (F0\<inter>S)) = sum g F\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   138
        by (intro sum.mono_neutral_cong) (use that \<open>finite F0\<close> F0'_def assms in auto)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   139
      finally show ?thesis .
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   140
    qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   141
    with \<open>F0' \<subseteq> T\<close> \<open>finite F0'\<close> show \<open>eventually P (filtermap (sum g) (finite_subsets_at_top T))\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   142
      by (metis (no_types, lifting) eventually_filtermap eventually_finite_subsets_at_top)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   143
  next
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   144
    assume \<open>eventually P (filtermap (sum g) (finite_subsets_at_top T))\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   145
    then obtain F0 where \<open>finite F0\<close> and \<open>F0 \<subseteq> T\<close> and F0_P: \<open>\<And>F. finite F \<Longrightarrow> F \<subseteq> T \<Longrightarrow> F \<supseteq> F0 \<Longrightarrow> P (sum g F)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   146
      by (metis (no_types, lifting) eventually_filtermap eventually_finite_subsets_at_top)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   147
    define F0' where \<open>F0' = F0 \<inter> S\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   148
    have [simp]: \<open>finite F0'\<close> \<open>F0' \<subseteq> S\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   149
      by (simp_all add: F0'_def \<open>finite F0\<close>)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   150
    have \<open>P (sum f F)\<close> if \<open>finite F\<close> \<open>F \<subseteq> S\<close> \<open>F \<supseteq> F0'\<close> for F
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   151
    proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   152
      have \<open>P (sum g ((F\<inter>T) \<union> (F0\<inter>T)))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   153
        by (intro F0_P) (use \<open>F0 \<subseteq> T\<close> \<open>finite F0\<close> that in auto)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   154
      also have \<open>sum g ((F\<inter>T) \<union> (F0\<inter>T)) = sum f F\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   155
        by (intro sum.mono_neutral_cong) (use that \<open>finite F0\<close> F0'_def assms in auto)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   156
      finally show ?thesis .
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   157
    qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   158
    with \<open>F0' \<subseteq> S\<close> \<open>finite F0'\<close> show \<open>eventually P (filtermap (sum f) (finite_subsets_at_top S))\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   159
      by (metis (no_types, lifting) eventually_filtermap eventually_finite_subsets_at_top)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   160
  qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   161
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   162
  then have tendsto_x: "(sum f \<longlongrightarrow> x) (finite_subsets_at_top S) \<longleftrightarrow> (sum g \<longlongrightarrow> x) (finite_subsets_at_top T)" for x
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   163
    by (simp add: le_filter_def filterlim_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   164
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   165
  then show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   166
    by (simp add: has_sum_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   167
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   168
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   169
lemma summable_on_cong_neutral: 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   170
  fixes f g :: \<open>'a \<Rightarrow> 'b::{comm_monoid_add, topological_space}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   171
  assumes \<open>\<And>x. x\<in>T-S \<Longrightarrow> g x = 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   172
  assumes \<open>\<And>x. x\<in>S-T \<Longrightarrow> f x = 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   173
  assumes \<open>\<And>x. x\<in>S\<inter>T \<Longrightarrow> f x = g x\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   174
  shows "f summable_on S \<longleftrightarrow> g summable_on T"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   175
  using has_sum_cong_neutral[of T S g f, OF assms]
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   176
  by (simp add: summable_on_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   177
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   178
lemma infsum_cong_neutral: 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   179
  fixes f g :: \<open>'a \<Rightarrow> 'b::{comm_monoid_add, t2_space}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   180
  assumes \<open>\<And>x. x\<in>T-S \<Longrightarrow> g x = 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   181
  assumes \<open>\<And>x. x\<in>S-T \<Longrightarrow> f x = 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   182
  assumes \<open>\<And>x. x\<in>S\<inter>T \<Longrightarrow> f x = g x\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   183
  shows \<open>infsum f S = infsum g T\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   184
  by (smt (verit, best) assms has_sum_cong_neutral infsum_eqI')
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   185
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   186
lemma has_sum_cong: 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   187
  assumes "\<And>x. x\<in>A \<Longrightarrow> f x = g x"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   188
  shows "(f has_sum x) A \<longleftrightarrow> (g has_sum x) A"
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   189
  using assms by (intro has_sum_cong_neutral) auto
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   190
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   191
lemma summable_on_cong:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   192
  assumes "\<And>x. x\<in>A \<Longrightarrow> f x = g x"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   193
  shows "f summable_on A \<longleftrightarrow> g summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   194
  by (metis assms summable_on_def has_sum_cong)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   195
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   196
lemma infsum_cong:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   197
  assumes "\<And>x. x\<in>A \<Longrightarrow> f x = g x"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   198
  shows "infsum f A = infsum g A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   199
  using assms infsum_eqI' has_sum_cong by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   200
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   201
lemma summable_on_cofin_subset:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   202
  fixes f :: "'a \<Rightarrow> 'b::topological_ab_group_add"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   203
  assumes "f summable_on A" and [simp]: "finite F"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   204
  shows "f summable_on (A - F)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   205
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   206
  from assms(1) obtain x where lim_f: "(sum f \<longlongrightarrow> x) (finite_subsets_at_top A)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   207
    unfolding summable_on_def has_sum_def by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   208
  define F' where "F' = F\<inter>A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   209
  with assms have "finite F'" and "A-F = A-F'"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   210
    by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   211
  have "filtermap ((\<union>)F') (finite_subsets_at_top (A-F))
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   212
      \<le> finite_subsets_at_top A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   213
  proof (rule filter_leI)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   214
    fix P assume "eventually P (finite_subsets_at_top A)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   215
    then obtain X where [simp]: "finite X" and XA: "X \<subseteq> A" 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   216
      and P: "\<forall>Y. finite Y \<and> X \<subseteq> Y \<and> Y \<subseteq> A \<longrightarrow> P Y"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   217
      unfolding eventually_finite_subsets_at_top by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   218
    define X' where "X' = X-F"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   219
    hence [simp]: "finite X'" and [simp]: "X' \<subseteq> A-F"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   220
      using XA by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   221
    hence "finite Y \<and> X' \<subseteq> Y \<and> Y \<subseteq> A - F \<longrightarrow> P (F' \<union> Y)" for Y
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   222
      using P XA unfolding X'_def using F'_def \<open>finite F'\<close> by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   223
    thus "eventually P (filtermap ((\<union>) F') (finite_subsets_at_top (A - F)))"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   224
      unfolding eventually_filtermap eventually_finite_subsets_at_top
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   225
      by (rule_tac x=X' in exI, simp)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   226
  qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   227
  with lim_f have "(sum f \<longlongrightarrow> x) (filtermap ((\<union>)F') (finite_subsets_at_top (A-F)))"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   228
    using tendsto_mono by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   229
  have "((\<lambda>G. sum f (F' \<union> G)) \<longlongrightarrow> x) (finite_subsets_at_top (A - F))"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   230
    if "((sum f \<circ> (\<union>) F') \<longlongrightarrow> x) (finite_subsets_at_top (A - F))"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   231
    using that unfolding o_def by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   232
  hence "((\<lambda>G. sum f (F' \<union> G)) \<longlongrightarrow> x) (finite_subsets_at_top (A-F))"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   233
    using tendsto_compose_filtermap [symmetric]
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   234
    by (simp add: \<open>(sum f \<longlongrightarrow> x) (filtermap ((\<union>) F') (finite_subsets_at_top (A - F)))\<close> 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   235
        tendsto_compose_filtermap)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   236
  have "\<forall>Y. finite Y \<and> Y \<subseteq> A - F \<longrightarrow> sum f (F' \<union> Y) = sum f F' + sum f Y"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   237
    by (metis Diff_disjoint Int_Diff \<open>A - F = A - F'\<close> \<open>finite F'\<close> inf.orderE sum.union_disjoint)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   238
  hence "\<forall>\<^sub>F x in finite_subsets_at_top (A - F). sum f (F' \<union> x) = sum f F' + sum f x"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   239
    unfolding eventually_finite_subsets_at_top
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   240
    using exI [where x = "{}"]
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   241
    by (simp add: \<open>\<And>P. P {} \<Longrightarrow> \<exists>x. P x\<close>) 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   242
  hence "((\<lambda>G. sum f F' + sum f G) \<longlongrightarrow> x) (finite_subsets_at_top (A-F))"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   243
    using tendsto_cong [THEN iffD1 , rotated]
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   244
      \<open>((\<lambda>G. sum f (F' \<union> G)) \<longlongrightarrow> x) (finite_subsets_at_top (A - F))\<close> by fastforce
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   245
  hence "((\<lambda>G. sum f F' + sum f G) \<longlongrightarrow> sum f F' + (x-sum f F')) (finite_subsets_at_top (A-F))"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   246
    by simp
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   247
  hence "(sum f \<longlongrightarrow> x - sum f F') (finite_subsets_at_top (A-F))"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   248
    using tendsto_add_const_iff by blast    
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   249
  thus "f summable_on (A - F)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   250
    unfolding summable_on_def has_sum_def by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   251
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   252
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   253
lemma
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   254
  fixes f :: "'a \<Rightarrow> 'b::{topological_ab_group_add}"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   255
  assumes \<open>(f has_sum b) B\<close> and \<open>(f has_sum a) A\<close> and AB: "A \<subseteq> B"
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   256
  shows has_sum_Diff: "(f has_sum (b - a)) (B - A)"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   257
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   258
  have finite_subsets1:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   259
    "finite_subsets_at_top (B - A) \<le> filtermap (\<lambda>F. F - A) (finite_subsets_at_top B)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   260
  proof (rule filter_leI)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   261
    fix P assume "eventually P (filtermap (\<lambda>F. F - A) (finite_subsets_at_top B))"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   262
    then obtain X where "finite X" and "X \<subseteq> B" 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   263
      and P: "finite Y \<and> X \<subseteq> Y \<and> Y \<subseteq> B \<longrightarrow> P (Y - A)" for Y
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   264
      unfolding eventually_filtermap eventually_finite_subsets_at_top by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   265
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   266
    hence "finite (X-A)" and "X-A \<subseteq> B - A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   267
      by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   268
    moreover have "finite Y \<and> X-A \<subseteq> Y \<and> Y \<subseteq> B - A \<longrightarrow> P Y" for Y
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   269
      using P[where Y="Y\<union>X"] \<open>finite X\<close> \<open>X \<subseteq> B\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   270
      by (metis Diff_subset Int_Diff Un_Diff finite_Un inf.orderE le_sup_iff sup.orderE sup_ge2)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   271
    ultimately show "eventually P (finite_subsets_at_top (B - A))"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   272
      unfolding eventually_finite_subsets_at_top by meson
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   273
  qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   274
  have finite_subsets2: 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   275
    "filtermap (\<lambda>F. F \<inter> A) (finite_subsets_at_top B) \<le> finite_subsets_at_top A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   276
    apply (rule filter_leI)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   277
      using assms unfolding eventually_filtermap eventually_finite_subsets_at_top
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   278
      by (metis Int_subset_iff finite_Int inf_le2 subset_trans)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   279
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   280
  from assms(1) have limB: "(sum f \<longlongrightarrow> b) (finite_subsets_at_top B)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   281
    using has_sum_def by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   282
  from assms(2) have limA: "(sum f \<longlongrightarrow> a) (finite_subsets_at_top A)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   283
    using has_sum_def by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   284
  have "((\<lambda>F. sum f (F\<inter>A)) \<longlongrightarrow> a) (finite_subsets_at_top B)"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   285
  proof (subst asm_rl [of "(\<lambda>F. sum f (F\<inter>A)) = sum f \<circ> (\<lambda>F. F\<inter>A)"])
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   286
    show "(\<lambda>F. sum f (F \<inter> A)) = sum f \<circ> (\<lambda>F. F \<inter> A)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   287
      unfolding o_def by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   288
    show "((sum f \<circ> (\<lambda>F. F \<inter> A)) \<longlongrightarrow> a) (finite_subsets_at_top B)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   289
      unfolding o_def 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   290
      using tendsto_compose_filtermap finite_subsets2 limA tendsto_mono
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   291
        \<open>(\<lambda>F. sum f (F \<inter> A)) = sum f \<circ> (\<lambda>F. F \<inter> A)\<close> by fastforce
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   292
  qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   293
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   294
  with limB have "((\<lambda>F. sum f F - sum f (F\<inter>A)) \<longlongrightarrow> b - a) (finite_subsets_at_top B)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   295
    using tendsto_diff by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   296
  have "sum f X - sum f (X \<inter> A) = sum f (X - A)" if "finite X" and "X \<subseteq> B" for X :: "'a set"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   297
    using that by (metis add_diff_cancel_left' sum.Int_Diff)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   298
  hence "\<forall>\<^sub>F x in finite_subsets_at_top B. sum f x - sum f (x \<inter> A) = sum f (x - A)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   299
    by (rule eventually_finite_subsets_at_top_weakI)  
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   300
  hence "((\<lambda>F. sum f (F-A)) \<longlongrightarrow> b - a) (finite_subsets_at_top B)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   301
    using tendsto_cong [THEN iffD1 , rotated]
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   302
      \<open>((\<lambda>F. sum f F - sum f (F \<inter> A)) \<longlongrightarrow> b - a) (finite_subsets_at_top B)\<close> by fastforce
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   303
  hence "(sum f \<longlongrightarrow> b - a) (filtermap (\<lambda>F. F-A) (finite_subsets_at_top B))"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   304
    by (subst tendsto_compose_filtermap[symmetric], simp add: o_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   305
  thus ?thesis
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   306
    using finite_subsets1 has_sum_def tendsto_mono by blast
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   307
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   308
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   309
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   310
lemma
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   311
  fixes f :: "'a \<Rightarrow> 'b::{topological_ab_group_add}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   312
  assumes "f summable_on B" and "f summable_on A" and "A \<subseteq> B"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   313
  shows summable_on_Diff: "f summable_on (B-A)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   314
  by (meson assms summable_on_def has_sum_Diff)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   315
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   316
lemma
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   317
  fixes f :: "'a \<Rightarrow> 'b::{topological_ab_group_add,t2_space}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   318
  assumes "f summable_on B" and "f summable_on A" and AB: "A \<subseteq> B"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   319
  shows infsum_Diff: "infsum f (B - A) = infsum f B - infsum f A"
74639
f831b6e589dc tuned proofs -- avoid z3, which is unavailable on arm64-linux;
wenzelm
parents: 74475
diff changeset
   320
  by (metis AB assms has_sum_Diff infsumI summable_on_def)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   321
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   322
lemma has_sum_mono_neutral:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   323
  fixes f :: "'a\<Rightarrow>'b::{ordered_comm_monoid_add,linorder_topology}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   324
  (* Does this really require a linorder topology? (Instead of order topology.) *)
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   325
  assumes \<open>(f has_sum a) A\<close> and "(g has_sum b) B"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   326
  assumes \<open>\<And>x. x \<in> A\<inter>B \<Longrightarrow> f x \<le> g x\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   327
  assumes \<open>\<And>x. x \<in> A-B \<Longrightarrow> f x \<le> 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   328
  assumes \<open>\<And>x. x \<in> B-A \<Longrightarrow> g x \<ge> 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   329
  shows "a \<le> b"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   330
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   331
  define f' g' where \<open>f' x = (if x \<in> A then f x else 0)\<close> and \<open>g' x = (if x \<in> B then g x else 0)\<close> for x
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   332
  have [simp]: \<open>f summable_on A\<close> \<open>g summable_on B\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   333
    using assms(1,2) summable_on_def by auto
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   334
  have \<open>(f' has_sum a) (A\<union>B)\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   335
    by (smt (verit, best) DiffE IntE Un_iff f'_def assms(1) has_sum_cong_neutral)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   336
  then have f'_lim: \<open>(sum f' \<longlongrightarrow> a) (finite_subsets_at_top (A\<union>B))\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   337
    by (meson has_sum_def)
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   338
  have \<open>(g' has_sum b) (A\<union>B)\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   339
  by (smt (verit, best) DiffD1 DiffD2 IntE UnCI g'_def assms(2) has_sum_cong_neutral)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   340
  then have g'_lim: \<open>(sum g' \<longlongrightarrow> b) (finite_subsets_at_top (A\<union>B))\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   341
    using has_sum_def by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   342
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   343
  have "\<And>X i. \<lbrakk>X \<subseteq> A \<union> B; i \<in> X\<rbrakk> \<Longrightarrow> f' i \<le> g' i"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   344
    using assms by (auto simp: f'_def g'_def)
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   345
  then have \<open>\<forall>\<^sub>F x in finite_subsets_at_top (A \<union> B). sum f' x \<le> sum g' x\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   346
    by (intro eventually_finite_subsets_at_top_weakI sum_mono)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   347
  then show ?thesis
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   348
    using f'_lim finite_subsets_at_top_neq_bot g'_lim tendsto_le by blast
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   349
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   350
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   351
lemma infsum_mono_neutral:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   352
  fixes f :: "'a\<Rightarrow>'b::{ordered_comm_monoid_add,linorder_topology}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   353
  assumes "f summable_on A" and "g summable_on B"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   354
  assumes \<open>\<And>x. x \<in> A\<inter>B \<Longrightarrow> f x \<le> g x\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   355
  assumes \<open>\<And>x. x \<in> A-B \<Longrightarrow> f x \<le> 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   356
  assumes \<open>\<And>x. x \<in> B-A \<Longrightarrow> g x \<ge> 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   357
  shows "infsum f A \<le> infsum g B"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   358
  by (smt (verit, best) assms has_sum_infsum has_sum_mono_neutral)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   359
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   360
lemma has_sum_mono:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   361
  fixes f :: "'a\<Rightarrow>'b::{ordered_comm_monoid_add,linorder_topology}"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   362
  assumes "(f has_sum x) A" and "(g has_sum y) A"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   363
  assumes \<open>\<And>x. x \<in> A \<Longrightarrow> f x \<le> g x\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   364
  shows "x \<le> y"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   365
  using assms has_sum_mono_neutral by force
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   366
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   367
lemma infsum_mono:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   368
  fixes f :: "'a\<Rightarrow>'b::{ordered_comm_monoid_add,linorder_topology}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   369
  assumes "f summable_on A" and "g summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   370
  assumes \<open>\<And>x. x \<in> A \<Longrightarrow> f x \<le> g x\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   371
  shows "infsum f A \<le> infsum g A"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   372
  by (meson assms has_sum_infsum has_sum_mono)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   373
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   374
lemma has_sum_finite[simp]:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   375
  assumes "finite F"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   376
  shows "(f has_sum (sum f F)) F"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   377
  using assms
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   378
  by (auto intro: tendsto_Lim simp: finite_subsets_at_top_finite infsum_def has_sum_def principal_eq_bot_iff)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   379
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   380
lemma summable_on_finite[simp]:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   381
  fixes f :: \<open>'a \<Rightarrow> 'b::{comm_monoid_add,topological_space}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   382
  assumes "finite F"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   383
  shows "f summable_on F"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   384
  using assms summable_on_def has_sum_finite by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   385
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   386
lemma infsum_finite[simp]:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   387
  assumes "finite F"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   388
  shows "infsum f F = sum f F"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   389
  by (simp add: assms infsumI)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   390
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   391
lemma has_sum_finite_approximation:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   392
  fixes f :: "'a \<Rightarrow> 'b::{comm_monoid_add,metric_space}"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   393
  assumes "(f has_sum x) A" and "\<epsilon> > 0"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   394
  shows "\<exists>F. finite F \<and> F \<subseteq> A \<and> dist (sum f F) x \<le> \<epsilon>"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   395
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   396
  have "(sum f \<longlongrightarrow> x) (finite_subsets_at_top A)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   397
    by (meson assms(1) has_sum_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   398
  hence *: "\<forall>\<^sub>F F in (finite_subsets_at_top A). dist (sum f F) x < \<epsilon>"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   399
    using assms(2) by (rule tendstoD)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   400
  thus ?thesis
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   401
    unfolding eventually_finite_subsets_at_top by fastforce
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   402
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   403
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   404
lemma infsum_finite_approximation:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   405
  fixes f :: "'a \<Rightarrow> 'b::{comm_monoid_add,metric_space}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   406
  assumes "f summable_on A" and "\<epsilon> > 0"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   407
  shows "\<exists>F. finite F \<and> F \<subseteq> A \<and> dist (sum f F) (infsum f A) \<le> \<epsilon>"
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   408
proof -
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   409
  from assms have "(f has_sum (infsum f A)) A"
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   410
    by (simp add: summable_iff_has_sum_infsum)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   411
  from this and \<open>\<epsilon> > 0\<close> show ?thesis
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   412
    by (rule has_sum_finite_approximation)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   413
qed
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   414
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   415
lemma abs_summable_summable:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   416
  fixes f :: \<open>'a \<Rightarrow> 'b :: banach\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   417
  assumes \<open>f abs_summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   418
  shows \<open>f summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   419
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   420
  from assms obtain L where lim: \<open>(sum (\<lambda>x. norm (f x)) \<longlongrightarrow> L) (finite_subsets_at_top A)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   421
    unfolding has_sum_def summable_on_def by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   422
  then have *: \<open>cauchy_filter (filtermap (sum (\<lambda>x. norm (f x))) (finite_subsets_at_top A))\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   423
    by (auto intro!: nhds_imp_cauchy_filter simp: filterlim_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   424
  have \<open>\<exists>P. eventually P (finite_subsets_at_top A) \<and>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   425
              (\<forall>F F'. P F \<and> P F' \<longrightarrow> dist (sum f F) (sum f F') < e)\<close> if \<open>e>0\<close> for e
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   426
  proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   427
    define d P where \<open>d = e/4\<close> and \<open>P F \<longleftrightarrow> finite F \<and> F \<subseteq> A \<and> dist (sum (\<lambda>x. norm (f x)) F) L < d\<close> for F
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   428
    then have \<open>d > 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   429
      by (simp add: d_def that)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   430
    have ev_P: \<open>eventually P (finite_subsets_at_top A)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   431
      using lim
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   432
      by (auto simp add: P_def[abs_def] \<open>0 < d\<close> eventually_conj_iff eventually_finite_subsets_at_top_weakI tendsto_iff)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   433
    
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   434
    moreover have \<open>dist (sum f F1) (sum f F2) < e\<close> if \<open>P F1\<close> and \<open>P F2\<close> for F1 F2
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   435
    proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   436
      from ev_P
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   437
      obtain F' where \<open>finite F'\<close> and \<open>F' \<subseteq> A\<close> and P_sup_F': \<open>finite F \<and> F \<supseteq> F' \<and> F \<subseteq> A \<Longrightarrow> P F\<close> for F
74639
f831b6e589dc tuned proofs -- avoid z3, which is unavailable on arm64-linux;
wenzelm
parents: 74475
diff changeset
   438
        by atomize_elim (simp add: eventually_finite_subsets_at_top)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   439
      define F where \<open>F = F' \<union> F1 \<union> F2\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   440
      have \<open>finite F\<close> and \<open>F \<subseteq> A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   441
        using F_def P_def[abs_def] that \<open>finite F'\<close> \<open>F' \<subseteq> A\<close> by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   442
      have dist_F: \<open>dist (sum (\<lambda>x. norm (f x)) F) L < d\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   443
        by (metis F_def \<open>F \<subseteq> A\<close> P_def P_sup_F' \<open>finite F\<close> le_supE order_refl)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   444
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   445
      have dist_F_subset: \<open>dist (sum f F) (sum f F') < 2*d\<close> if F': \<open>F' \<subseteq> F\<close> \<open>P F'\<close> for F'
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   446
      proof -
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   447
        have \<open>dist (sum f F) (sum f F') = norm (sum f (F-F'))\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   448
          unfolding dist_norm using \<open>finite F\<close> F' by (subst sum_diff) auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   449
        also have \<open>\<dots> \<le> norm (\<Sum>x\<in>F-F'. norm (f x))\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   450
          by (rule order.trans[OF sum_norm_le[OF order.refl]]) auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   451
        also have \<open>\<dots> = dist (\<Sum>x\<in>F. norm (f x)) (\<Sum>x\<in>F'. norm (f x))\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   452
          unfolding dist_norm using \<open>finite F\<close> F' by (subst sum_diff) auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   453
        also have \<open>\<dots> < 2 * d\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   454
          using dist_F F' unfolding P_def dist_norm real_norm_def by linarith
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   455
        finally show \<open>dist (sum f F) (sum f F') < 2*d\<close> .
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   456
      qed
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   457
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   458
      have \<open>dist (sum f F1) (sum f F2) \<le> dist (sum f F) (sum f F1) + dist (sum f F) (sum f F2)\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   459
        by (rule dist_triangle3)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   460
      also have \<open>\<dots> < 2 * d + 2 * d\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   461
        by (intro add_strict_mono dist_F_subset that) (auto simp: F_def)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   462
      also have \<open>\<dots> \<le> e\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   463
        by (auto simp: d_def)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   464
      finally show \<open>dist (sum f F1) (sum f F2) < e\<close> .
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   465
    qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   466
    then show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   467
      using ev_P by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   468
  qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   469
  then have \<open>cauchy_filter (filtermap (sum f) (finite_subsets_at_top A))\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   470
    by (simp add: cauchy_filter_metric_filtermap)
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   471
  moreover have "complete (UNIV::'b set)"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   472
    by (meson Cauchy_convergent UNIV_I complete_def convergent_def)
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   473
  ultimately obtain L' where \<open>(sum f \<longlongrightarrow> L') (finite_subsets_at_top A)\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   474
    using complete_uniform[where S=UNIV] by (force simp add: filterlim_def)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   475
  then show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   476
    using summable_on_def has_sum_def by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   477
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   478
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   479
text \<open>The converse of @{thm [source] abs_summable_summable} does not hold:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   480
  Consider the Hilbert space of square-summable sequences.
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   481
  Let $e_i$ denote the sequence with 1 in the $i$th position and 0 elsewhere.
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   482
  Let $f(i) := e_i/i$ for $i\geq1$. We have \<^term>\<open>\<not> f abs_summable_on UNIV\<close> because $\lVert f(i)\rVert=1/i$
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   483
  and thus the sum over $\lVert f(i)\rVert$ diverges. On the other hand, we have \<^term>\<open>f summable_on UNIV\<close>;
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   484
  the limit is the sequence with $1/i$ in the $i$th position.
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   485
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   486
  (We have not formalized this separating example here because to the best of our knowledge,
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   487
  this Hilbert space has not been formalized in Isabelle/HOL yet.)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   488
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   489
lemma norm_has_sum_bound:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   490
  fixes f :: "'b \<Rightarrow> 'a::real_normed_vector"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   491
    and A :: "'b set"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   492
  assumes "((\<lambda>x. norm (f x)) has_sum n) A"
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   493
  assumes "(f has_sum a) A"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   494
  shows "norm a \<le> n"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   495
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   496
  have "norm a \<le> n + \<epsilon>" if "\<epsilon>>0" for \<epsilon>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   497
  proof-
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   498
    have "\<exists>F. norm (a - sum f F) \<le> \<epsilon> \<and> finite F \<and> F \<subseteq> A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   499
      using has_sum_finite_approximation[where A=A and f=f and \<epsilon>="\<epsilon>"] assms \<open>0 < \<epsilon>\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   500
      by (metis dist_commute dist_norm)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   501
    then obtain F where "norm (a - sum f F) \<le> \<epsilon>"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   502
      and "finite F" and "F \<subseteq> A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   503
      by (simp add: atomize_elim)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   504
    hence "norm a \<le> norm (sum f F) + \<epsilon>"
74642
8af77cb50c6d tuned proofs -- avoid z3, which is unavailable on arm64-linux;
wenzelm
parents: 74639
diff changeset
   505
      by (metis add.commute diff_add_cancel dual_order.refl norm_triangle_mono)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   506
    also have "\<dots> \<le> sum (\<lambda>x. norm (f x)) F + \<epsilon>"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   507
      using norm_sum by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   508
    also have "\<dots> \<le> n + \<epsilon>"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   509
    proof (intro add_right_mono [OF has_sum_mono_neutral])
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   510
      show "((\<lambda>x. norm (f x)) has_sum (\<Sum>x\<in>F. norm (f x))) F"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   511
        by (simp add: \<open>finite F\<close>)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   512
    qed (use \<open>F \<subseteq> A\<close> assms in auto)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   513
    finally show ?thesis 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   514
      by assumption
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   515
  qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   516
  thus ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   517
    using linordered_field_class.field_le_epsilon by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   518
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   519
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   520
lemma norm_infsum_bound:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   521
  fixes f :: "'b \<Rightarrow> 'a::real_normed_vector"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   522
    and A :: "'b set"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   523
  assumes "f abs_summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   524
  shows "norm (infsum f A) \<le> infsum (\<lambda>x. norm (f x)) A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   525
proof (cases "f summable_on A")
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   526
  case True
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   527
  have "((\<lambda>x. norm (f x)) has_sum (\<Sum>\<^sub>\<infinity>x\<in>A. norm (f x))) A"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   528
    by (simp add: assms)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   529
  then show ?thesis
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   530
    by (metis True has_sum_infsum norm_has_sum_bound)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   531
next
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   532
  case False
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   533
  obtain t where t_def: "(sum (\<lambda>x. norm (f x)) \<longlongrightarrow> t) (finite_subsets_at_top A)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   534
    using assms unfolding summable_on_def has_sum_def by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   535
  have sumpos: "sum (\<lambda>x. norm (f x)) X \<ge> 0"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   536
    for X
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   537
    by (simp add: sum_nonneg)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   538
  have tgeq0:"t \<ge> 0"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   539
  proof(rule ccontr)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   540
    define S::"real set" where "S = {s. s < 0}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   541
    assume "\<not> 0 \<le> t"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   542
    hence "t < 0" by simp
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   543
    hence "t \<in> S"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   544
      unfolding S_def by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   545
    moreover have "open S"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   546
      by (metis S_def lessThan_def open_real_lessThan)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   547
    ultimately have "\<forall>\<^sub>F X in finite_subsets_at_top A. (\<Sum>x\<in>X. norm (f x)) \<in> S"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   548
      using t_def unfolding tendsto_def by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   549
    hence "\<exists>X. (\<Sum>x\<in>X. norm (f x)) \<in> S"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   550
      by (metis (no_types, lifting) eventually_mono filterlim_iff finite_subsets_at_top_neq_bot tendsto_Lim)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   551
    then obtain X where "(\<Sum>x\<in>X. norm (f x)) \<in> S"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   552
      by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   553
    hence "(\<Sum>x\<in>X. norm (f x)) < 0"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   554
      unfolding S_def by auto      
74642
8af77cb50c6d tuned proofs -- avoid z3, which is unavailable on arm64-linux;
wenzelm
parents: 74639
diff changeset
   555
    thus False by (simp add: leD sumpos)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   556
  qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   557
  have "\<exists>!h. (sum (\<lambda>x. norm (f x)) \<longlongrightarrow> h) (finite_subsets_at_top A)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   558
    using t_def finite_subsets_at_top_neq_bot tendsto_unique by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   559
  hence "t = (Topological_Spaces.Lim (finite_subsets_at_top A) (sum (\<lambda>x. norm (f x))))"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   560
    using t_def unfolding Topological_Spaces.Lim_def
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   561
    by (metis the_equality)     
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   562
  hence "Lim (finite_subsets_at_top A) (sum (\<lambda>x. norm (f x))) \<ge> 0"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   563
    using tgeq0 by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   564
  thus ?thesis unfolding infsum_def 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   565
    using False by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   566
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   567
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   568
lemma infsum_tendsto:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   569
  assumes \<open>f summable_on S\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   570
  shows \<open>((\<lambda>F. sum f F) \<longlongrightarrow> infsum f S) (finite_subsets_at_top S)\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   571
  using assms has_sum_def has_sum_infsum by blast
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   572
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   573
lemma has_sum_0: 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   574
  assumes \<open>\<And>x. x\<in>M \<Longrightarrow> f x = 0\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   575
  shows \<open>(f has_sum 0) M\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   576
  by (metis assms finite.intros(1) has_sum_cong has_sum_cong_neutral has_sum_finite sum.neutral_const)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   577
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   578
lemma summable_on_0:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   579
  assumes \<open>\<And>x. x\<in>M \<Longrightarrow> f x = 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   580
  shows \<open>f summable_on M\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   581
  using assms summable_on_def has_sum_0 by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   582
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   583
lemma infsum_0:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   584
  assumes \<open>\<And>x. x\<in>M \<Longrightarrow> f x = 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   585
  shows \<open>infsum f M = 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   586
  by (metis assms finite_subsets_at_top_neq_bot infsum_def has_sum_0 has_sum_def tendsto_Lim)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   587
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   588
text \<open>Variants of @{thm [source] infsum_0} etc. suitable as simp-rules\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   589
lemma infsum_0_simp[simp]: \<open>infsum (\<lambda>_. 0) M = 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   590
  by (simp_all add: infsum_0)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   591
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   592
lemma summable_on_0_simp[simp]: \<open>(\<lambda>_. 0) summable_on M\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   593
  by (simp_all add: summable_on_0)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   594
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   595
lemma has_sum_0_simp[simp]: \<open>((\<lambda>_. 0) has_sum 0) M\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   596
  by (simp_all add: has_sum_0)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   597
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   598
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   599
lemma has_sum_add:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   600
  fixes f g :: "'a \<Rightarrow> 'b::{topological_comm_monoid_add}"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   601
  assumes \<open>(f has_sum a) A\<close>
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   602
  assumes \<open>(g has_sum b) A\<close>
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   603
  shows \<open>((\<lambda>x. f x + g x) has_sum (a + b)) A\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   604
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   605
  from assms have lim_f: \<open>(sum f \<longlongrightarrow> a)  (finite_subsets_at_top A)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   606
    and lim_g: \<open>(sum g \<longlongrightarrow> b)  (finite_subsets_at_top A)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   607
    by (simp_all add: has_sum_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   608
  then have lim: \<open>(sum (\<lambda>x. f x + g x) \<longlongrightarrow> a + b) (finite_subsets_at_top A)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   609
    unfolding sum.distrib by (rule tendsto_add)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   610
  then show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   611
    by (simp_all add: has_sum_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   612
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   613
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   614
lemma summable_on_add:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   615
  fixes f g :: "'a \<Rightarrow> 'b::{topological_comm_monoid_add}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   616
  assumes \<open>f summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   617
  assumes \<open>g summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   618
  shows \<open>(\<lambda>x. f x + g x) summable_on A\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   619
  by (metis (full_types) assms summable_on_def has_sum_add)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   620
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   621
lemma infsum_add:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   622
  fixes f g :: "'a \<Rightarrow> 'b::{topological_comm_monoid_add, t2_space}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   623
  assumes \<open>f summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   624
  assumes \<open>g summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   625
  shows \<open>infsum (\<lambda>x. f x + g x) A = infsum f A + infsum g A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   626
proof -
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   627
  have \<open>((\<lambda>x. f x + g x) has_sum (infsum f A + infsum g A)) A\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   628
    by (simp add: assms has_sum_add)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   629
  then show ?thesis
74639
f831b6e589dc tuned proofs -- avoid z3, which is unavailable on arm64-linux;
wenzelm
parents: 74475
diff changeset
   630
    using infsumI by blast
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   631
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   632
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   633
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   634
lemma has_sum_Un_disjoint:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   635
  fixes f :: "'a \<Rightarrow> 'b::topological_comm_monoid_add"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   636
  assumes "(f has_sum a) A"
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   637
  assumes "(f has_sum b) B"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   638
  assumes disj: "A \<inter> B = {}"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   639
  shows \<open>(f has_sum (a + b)) (A \<union> B)\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   640
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   641
  define fA fB where \<open>fA x = (if x \<in> A then f x else 0)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   642
    and \<open>fB x = (if x \<notin> A then f x else 0)\<close> for x
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   643
  have fA: \<open>(fA has_sum a) (A \<union> B)\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   644
    by (smt (verit, ccfv_SIG) DiffD1 DiffD2 UnCI fA_def assms(1) has_sum_cong_neutral inf_sup_absorb)
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   645
  have fB: \<open>(fB has_sum b) (A \<union> B)\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   646
    by (smt (verit, best) DiffD1 DiffD2 IntE Un_iff fB_def assms(2) disj disjoint_iff has_sum_cong_neutral)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   647
  have fAB: \<open>f x = fA x + fB x\<close> for x
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   648
    unfolding fA_def fB_def by simp
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   649
  show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   650
    unfolding fAB
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   651
    using fA fB by (rule has_sum_add)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   652
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   653
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   654
lemma summable_on_Un_disjoint:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   655
  fixes f :: "'a \<Rightarrow> 'b::topological_comm_monoid_add"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   656
  assumes "f summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   657
  assumes "f summable_on B"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   658
  assumes disj: "A \<inter> B = {}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   659
  shows \<open>f summable_on (A \<union> B)\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   660
  by (meson assms disj summable_on_def has_sum_Un_disjoint)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   661
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   662
lemma infsum_Un_disjoint:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   663
  fixes f :: "'a \<Rightarrow> 'b::{topological_comm_monoid_add, t2_space}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   664
  assumes "f summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   665
  assumes "f summable_on B"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   666
  assumes disj: "A \<inter> B = {}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   667
  shows \<open>infsum f (A \<union> B) = infsum f A + infsum f B\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   668
  by (intro infsumI has_sum_Un_disjoint has_sum_infsum assms)  
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   669
75462
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   670
lemma norm_summable_imp_has_sum:
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   671
  fixes f :: "nat \<Rightarrow> 'a :: banach"
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   672
  assumes "summable (\<lambda>n. norm (f n))" and "f sums S"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   673
  shows   "(f has_sum S) (UNIV :: nat set)"
75462
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   674
  unfolding has_sum_def tendsto_iff eventually_finite_subsets_at_top
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   675
proof clarsimp
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   676
  fix \<epsilon>::real 
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   677
  assume "\<epsilon> > 0"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   678
  from assms obtain S' where S': "(\<lambda>n. norm (f n)) sums S'"
75462
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   679
    by (auto simp: summable_def)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   680
  with \<open>\<epsilon> > 0\<close> obtain N where N: "\<And>n. n \<ge> N \<Longrightarrow> \<bar>S' - (\<Sum>i<n. norm (f i))\<bar> < \<epsilon>"
75462
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   681
    by (auto simp: tendsto_iff eventually_at_top_linorder sums_def dist_norm abs_minus_commute)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   682
  have "dist (sum f Y) S < \<epsilon>" if "finite Y" "{..<N} \<subseteq> Y" for Y
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   683
  proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   684
    from that have "(\<lambda>n. if n \<in> Y then 0 else f n) sums (S - sum f Y)"
75462
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   685
      by (intro sums_If_finite_set'[OF \<open>f sums S\<close>]) (auto simp: sum_negf)
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   686
    hence "S - sum f Y = (\<Sum>n. if n \<in> Y then 0 else f n)"
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   687
      by (simp add: sums_iff)
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   688
    also have "norm \<dots> \<le> (\<Sum>n. norm (if n \<in> Y then 0 else f n))"
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   689
      by (rule summable_norm[OF summable_comparison_test'[OF assms(1)]]) auto
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   690
    also have "\<dots> \<le> (\<Sum>n. if n < N then 0 else norm (f n))"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   691
      using that by (intro suminf_le summable_comparison_test'[OF assms(1)]) auto
75462
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   692
    also have "(\<lambda>n. if n \<in> {..<N} then 0 else norm (f n)) sums (S' - (\<Sum>i<N. norm (f i)))" 
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   693
      by (intro sums_If_finite_set'[OF S']) (auto simp: sum_negf)
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   694
    hence "(\<Sum>n. if n < N then 0 else norm (f n)) = S' - (\<Sum>i<N. norm (f i))"
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   695
      by (simp add: sums_iff)
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   696
    also have "S' - (\<Sum>i<N. norm (f i)) \<le> \<bar>S' - (\<Sum>i<N. norm (f i))\<bar>" by simp
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   697
    also have "\<dots> < \<epsilon>" by (rule N) auto
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   698
    finally show ?thesis by (simp add: dist_norm norm_minus_commute)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   699
  qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   700
  then show "\<exists>X. finite X \<and> (\<forall>Y. finite Y \<and> X \<subseteq> Y \<longrightarrow> dist (sum f Y) S < \<epsilon>)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   701
    by (meson finite_lessThan subset_UNIV)
75462
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   702
qed
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   703
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   704
lemma norm_summable_imp_summable_on:
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   705
  fixes f :: "nat \<Rightarrow> 'a :: banach"
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   706
  assumes "summable (\<lambda>n. norm (f n))"
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   707
  shows   "f summable_on UNIV"
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   708
  using norm_summable_imp_has_sum[OF assms, of "suminf f"] assms
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 74791
diff changeset
   709
  by (auto simp: sums_iff summable_on_def dest: summable_norm_cancel)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   710
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   711
text \<open>The following lemma indeed needs a complete space (as formalized by the premise \<^term>\<open>complete UNIV\<close>).
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   712
  The following two counterexamples show this:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   713
  \begin{itemize}
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   714
  \item Consider the real vector space $V$ of sequences with finite support, and with the $\ell_2$-norm (sum of squares).
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   715
      Let $e_i$ denote the sequence with a $1$ at position $i$.
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   716
      Let $f : \mathbb Z \to V$ be defined as $f(n) := e_{\lvert n\rvert} / n$ (with $f(0) := 0$).
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   717
      We have that $\sum_{n\in\mathbb Z} f(n) = 0$ (it even converges absolutely). 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   718
      But $\sum_{n\in\mathbb N} f(n)$ does not exist (it would converge against a sequence with infinite support).
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   719
  
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   720
  \item Let $f$ be a positive rational valued function such that $\sum_{x\in B} f(x)$ is $\sqrt 2$ and $\sum_{x\in A} f(x)$ is 1 (over the reals, with $A\subseteq B$).
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   721
      Then $\sum_{x\in B} f(x)$ does not exist over the rationals. But $\sum_{x\in A} f(x)$ exists.
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   722
  \end{itemize}
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   723
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   724
  The lemma also requires uniform continuity of the addition. And example of a topological group with continuous 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   725
  but not uniformly continuous addition would be the positive reals with the usual multiplication as the addition.
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   726
  We do not know whether the lemma would also hold for such topological groups.\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   727
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   728
lemma summable_on_subset_aux:
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   729
  fixes A B and f :: \<open>'a \<Rightarrow> 'b::{ab_group_add, uniform_space}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   730
  assumes \<open>complete (UNIV :: 'b set)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   731
  assumes plus_cont: \<open>uniformly_continuous_on UNIV (\<lambda>(x::'b,y). x+y)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   732
  assumes \<open>f summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   733
  assumes \<open>B \<subseteq> A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   734
  shows \<open>f summable_on B\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   735
proof -
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   736
  let ?filter_fB = \<open>filtermap (sum f) (finite_subsets_at_top B)\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   737
  from \<open>f summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   738
  obtain S where \<open>(sum f \<longlongrightarrow> S) (finite_subsets_at_top A)\<close> (is \<open>(sum f \<longlongrightarrow> S) ?filter_A\<close>)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   739
    using summable_on_def has_sum_def by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   740
  then have cauchy_fA: \<open>cauchy_filter (filtermap (sum f) (finite_subsets_at_top A))\<close> (is \<open>cauchy_filter ?filter_fA\<close>)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   741
    by (auto intro!: nhds_imp_cauchy_filter simp: filterlim_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   742
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   743
  have \<open>cauchy_filter (filtermap (sum f) (finite_subsets_at_top B))\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   744
  proof (unfold cauchy_filter_def, rule filter_leI)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   745
    fix E :: \<open>('b\<times>'b) \<Rightarrow> bool\<close> assume \<open>eventually E uniformity\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   746
    then obtain E' where \<open>eventually E' uniformity\<close> and E'E'E: \<open>E' (x, y) \<longrightarrow> E' (y, z) \<longrightarrow> E (x, z)\<close> for x y z
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   747
      using uniformity_trans by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   748
    obtain D where \<open>eventually D uniformity\<close> and DE: \<open>D (x, y) \<Longrightarrow> E' (x+c, y+c)\<close> for x y c
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   749
      using plus_cont \<open>eventually E' uniformity\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   750
      unfolding uniformly_continuous_on_uniformity filterlim_def le_filter_def uniformity_prod_def
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   751
      by (auto simp: case_prod_beta eventually_filtermap eventually_prod_same uniformity_refl)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   752
    have DE': "E' (x, y)" if "D (x + c, y + c)" for x y c
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   753
      using DE[of "x + c" "y + c" "-c"] that by simp
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   754
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   755
    from \<open>eventually D uniformity\<close> and cauchy_fA have \<open>eventually D (?filter_fA \<times>\<^sub>F ?filter_fA)\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   756
      unfolding cauchy_filter_def le_filter_def by simp
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   757
    then obtain P1 P2
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   758
      where ev_P1: \<open>eventually (\<lambda>F. P1 (sum f F)) ?filter_A\<close> 
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   759
        and ev_P2: \<open>eventually (\<lambda>F. P2 (sum f F)) ?filter_A\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   760
        and P1P2E: \<open>P1 x \<Longrightarrow> P2 y \<Longrightarrow> D (x, y)\<close> for x y
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   761
      unfolding eventually_prod_filter eventually_filtermap
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   762
      by auto
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   763
    from ev_P1 obtain F1 where F1: \<open>finite F1\<close> \<open>F1 \<subseteq> A\<close> \<open>\<And>F. F\<supseteq>F1 \<Longrightarrow> finite F \<Longrightarrow> F\<subseteq>A \<Longrightarrow> P1 (sum f F)\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   764
      by (metis eventually_finite_subsets_at_top)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   765
    from ev_P2 obtain F2 where F2: \<open>finite F2\<close> \<open>F2 \<subseteq> A\<close> \<open>\<And>F. F\<supseteq>F2 \<Longrightarrow> finite F \<Longrightarrow> F\<subseteq>A \<Longrightarrow> P2 (sum f F)\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   766
      by (metis eventually_finite_subsets_at_top)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   767
    define F0 F0A F0B where \<open>F0 \<equiv> F1 \<union> F2\<close> and \<open>F0A \<equiv> F0 - B\<close> and \<open>F0B \<equiv> F0 \<inter> B\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   768
    have [simp]: \<open>finite F0\<close>  \<open>F0 \<subseteq> A\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   769
      using \<open>F1 \<subseteq> A\<close> \<open>F2 \<subseteq> A\<close> \<open>finite F1\<close> \<open>finite F2\<close> unfolding F0_def by blast+
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   770
 
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   771
    have *: "E' (sum f F1', sum f F2')"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   772
      if "F1'\<supseteq>F0B" "F2'\<supseteq>F0B" "finite F1'" "finite F2'" "F1'\<subseteq>B" "F2'\<subseteq>B" for F1' F2'
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   773
    proof (intro DE'[where c = "sum f F0A"] P1P2E)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   774
      have "P1 (sum f (F1' \<union> F0A))"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   775
        using that assms F1(1,2) F2(1,2) by (intro F1) (auto simp: F0A_def F0B_def F0_def)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   776
      thus "P1 (sum f F1' + sum f F0A)"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   777
        by (subst (asm) sum.union_disjoint) (use that in \<open>auto simp: F0A_def\<close>)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   778
    next
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   779
      have "P2 (sum f (F2' \<union> F0A))"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   780
        using that assms F1(1,2) F2(1,2) by (intro F2) (auto simp: F0A_def F0B_def F0_def)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   781
      thus "P2 (sum f F2' + sum f F0A)"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   782
        by (subst (asm) sum.union_disjoint) (use that in \<open>auto simp: F0A_def\<close>)      
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   783
    qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   784
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
   785
    have "eventually (\<lambda>x. E' (x, sum f F0B)) (filtermap (sum f) (finite_subsets_at_top B))"
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
   786
     and "eventually (\<lambda>x. E' (sum f F0B, x)) (filtermap (sum f) (finite_subsets_at_top B))"
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
   787
        unfolding eventually_filtermap eventually_finite_subsets_at_top
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
   788
        by (rule exI[of _ F0B]; use * in \<open>force simp: F0B_def\<close>)+
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
   789
      then 
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   790
    show \<open>eventually E (?filter_fB \<times>\<^sub>F ?filter_fB)\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   791
      unfolding eventually_prod_filter
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
   792
      using E'E'E by blast
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   793
  qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   794
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   795
  then obtain x where \<open>?filter_fB \<le> nhds x\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   796
    using cauchy_filter_complete_converges[of ?filter_fB UNIV] \<open>complete (UNIV :: _)\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   797
    by (auto simp: filtermap_bot_iff)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   798
  then have \<open>(sum f \<longlongrightarrow> x) (finite_subsets_at_top B)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   799
    by (auto simp: filterlim_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   800
  then show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   801
    by (auto simp: summable_on_def has_sum_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   802
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   803
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   804
text \<open>A special case of @{thm [source] summable_on_subset_aux} for Banach spaces with fewer premises.\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   805
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   806
lemma summable_on_subset_banach:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   807
  fixes A B and f :: \<open>'a \<Rightarrow> 'b::banach\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   808
  assumes \<open>f summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   809
  assumes \<open>B \<subseteq> A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   810
  shows \<open>f summable_on B\<close>
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
   811
  by (meson Cauchy_convergent UNIV_I assms complete_def convergent_def isUCont_plus summable_on_subset_aux)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   812
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   813
lemma has_sum_empty[simp]: \<open>(f has_sum 0) {}\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   814
  by (meson ex_in_conv has_sum_0)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   815
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   816
lemma summable_on_empty[simp]: \<open>f summable_on {}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   817
  by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   818
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   819
lemma infsum_empty[simp]: \<open>infsum f {} = 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   820
  by simp
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   821
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   822
lemma sum_has_sum:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   823
  fixes f :: "'a \<Rightarrow> 'b::topological_comm_monoid_add"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   824
  assumes \<open>finite A\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   825
  assumes \<open>\<And>a. a \<in> A \<Longrightarrow> (f has_sum (s a)) (B a)\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   826
  assumes \<open>\<And>a a'. a\<in>A \<Longrightarrow> a'\<in>A \<Longrightarrow> a\<noteq>a' \<Longrightarrow> B a \<inter> B a' = {}\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   827
  shows \<open>(f has_sum (sum s A)) (\<Union>a\<in>A. B a)\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   828
  using assms 
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   829
proof (induction)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   830
  case empty
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   831
  then show ?case 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   832
    by simp
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   833
next
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   834
  case (insert x A)
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   835
  have \<open>(f has_sum (s x)) (B x)\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   836
    by (simp add: insert.prems)
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   837
  moreover have IH: \<open>(f has_sum (sum s A)) (\<Union>a\<in>A. B a)\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   838
    using insert by simp
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   839
  ultimately have \<open>(f has_sum (s x + sum s A)) (B x \<union> (\<Union>a\<in>A. B a))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   840
    using insert by (intro has_sum_Un_disjoint) auto
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   841
  then show ?case
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   842
    using insert.hyps by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   843
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   844
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   845
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   846
lemma summable_on_finite_union_disjoint:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   847
  fixes f :: "'a \<Rightarrow> 'b::topological_comm_monoid_add"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   848
  assumes finite: \<open>finite A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   849
  assumes conv: \<open>\<And>a. a \<in> A \<Longrightarrow> f summable_on (B a)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   850
  assumes disj: \<open>\<And>a a'. a\<in>A \<Longrightarrow> a'\<in>A \<Longrightarrow> a\<noteq>a' \<Longrightarrow> B a \<inter> B a' = {}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   851
  shows \<open>f summable_on (\<Union>a\<in>A. B a)\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   852
  using sum_has_sum [of A f B] assms unfolding summable_on_def by metis
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   853
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   854
lemma sum_infsum:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   855
  fixes f :: "'a \<Rightarrow> 'b::{topological_comm_monoid_add, t2_space}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   856
  assumes finite: \<open>finite A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   857
  assumes conv: \<open>\<And>a. a \<in> A \<Longrightarrow> f summable_on (B a)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   858
  assumes disj: \<open>\<And>a a'. a\<in>A \<Longrightarrow> a'\<in>A \<Longrightarrow> a\<noteq>a' \<Longrightarrow> B a \<inter> B a' = {}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   859
  shows \<open>sum (\<lambda>a. infsum f (B a)) A = infsum f (\<Union>a\<in>A. B a)\<close>
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
   860
  by (metis (no_types, lifting) assms has_sum_infsum infsumI sum_has_sum)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   861
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   862
text \<open>The lemmas \<open>infsum_comm_additive_general\<close> and \<open>infsum_comm_additive\<close> (and variants) below both state that the infinite sum commutes with
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   863
  a continuous additive function. \<open>infsum_comm_additive_general\<close> is stated more for more general type classes
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   864
  at the expense of a somewhat less compact formulation of the premises.
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   865
  E.g., by avoiding the constant \<^const>\<open>additive\<close> which introduces an additional sort constraint
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   866
  (group instead of monoid). For example, extended reals (\<^typ>\<open>ereal\<close>, \<^typ>\<open>ennreal\<close>) are not covered
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   867
  by \<open>infsum_comm_additive\<close>.\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   868
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   869
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   870
lemma has_sum_comm_additive_general: 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   871
  fixes f :: \<open>'b :: {comm_monoid_add,topological_space} \<Rightarrow> 'c :: {comm_monoid_add,topological_space}\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   872
  assumes f_sum: \<open>\<And>F. finite F \<Longrightarrow> F \<subseteq> S \<Longrightarrow> sum (f \<circ> g) F = f (sum g F)\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   873
      \<comment> \<open>Not using \<^const>\<open>additive\<close> because it would add sort constraint \<^class>\<open>ab_group_add\<close>\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   874
  assumes cont: \<open>f \<midarrow>x\<rightarrow> f x\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   875
    \<comment> \<open>For \<^class>\<open>t2_space\<close>, this is equivalent to \<open>isCont f x\<close> by @{thm [source] isCont_def}.\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   876
  assumes infsum: \<open>(g has_sum x) S\<close>
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   877
  shows \<open>((f \<circ> g) has_sum (f x)) S\<close> 
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   878
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   879
  have \<open>(sum g \<longlongrightarrow> x) (finite_subsets_at_top S)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   880
    using infsum has_sum_def by blast
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   881
  then have \<open>((f \<circ> sum g) \<longlongrightarrow> f x) (finite_subsets_at_top S)\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   882
    by (meson cont filterlim_def tendsto_at_iff_tendsto_nhds tendsto_compose_filtermap tendsto_mono)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   883
  then have \<open>(sum (f \<circ> g) \<longlongrightarrow> f x) (finite_subsets_at_top S)\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   884
    using tendsto_cong f_sum
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   885
    by (simp add: Lim_transform_eventually eventually_finite_subsets_at_top_weakI)
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   886
  then show \<open>((f \<circ> g) has_sum (f x)) S\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   887
    using has_sum_def by blast 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   888
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   889
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   890
lemma summable_on_comm_additive_general:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   891
  fixes f :: \<open>'b :: {comm_monoid_add,topological_space} \<Rightarrow> 'c :: {comm_monoid_add,topological_space}\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   892
  assumes \<open>\<And>F. finite F \<Longrightarrow> F \<subseteq> S \<Longrightarrow> sum (f \<circ> g) F = f (sum g F)\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   893
    \<comment> \<open>Not using \<^const>\<open>additive\<close> because it would add sort constraint \<^class>\<open>ab_group_add\<close>\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   894
  assumes \<open>\<And>x. (g has_sum x) S \<Longrightarrow> f \<midarrow>x\<rightarrow> f x\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   895
    \<comment> \<open>For \<^class>\<open>t2_space\<close>, this is equivalent to \<open>isCont f x\<close> by @{thm [source] isCont_def}.\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   896
  assumes \<open>g summable_on S\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   897
  shows \<open>(f \<circ> g) summable_on S\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   898
  by (meson assms summable_on_def has_sum_comm_additive_general has_sum_def infsum_tendsto)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   899
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   900
lemma infsum_comm_additive_general:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   901
  fixes f :: \<open>'b :: {comm_monoid_add,t2_space} \<Rightarrow> 'c :: {comm_monoid_add,t2_space}\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   902
  assumes f_sum: \<open>\<And>F. finite F \<Longrightarrow> F \<subseteq> S \<Longrightarrow> sum (f \<circ> g) F = f (sum g F)\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   903
      \<comment> \<open>Not using \<^const>\<open>additive\<close> because it would add sort constraint \<^class>\<open>ab_group_add\<close>\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   904
  assumes \<open>isCont f (infsum g S)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   905
  assumes \<open>g summable_on S\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   906
  shows \<open>infsum (f \<circ> g) S = f (infsum g S)\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   907
  using assms
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   908
  by (intro infsumI has_sum_comm_additive_general has_sum_infsum) (auto simp: isCont_def)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   909
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   910
lemma has_sum_comm_additive: 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   911
  fixes f :: \<open>'b :: {ab_group_add,topological_space} \<Rightarrow> 'c :: {ab_group_add,topological_space}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   912
  assumes \<open>additive f\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   913
  assumes \<open>f \<midarrow>x\<rightarrow> f x\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   914
    \<comment> \<open>For \<^class>\<open>t2_space\<close>, this is equivalent to \<open>isCont f x\<close> by @{thm [source] isCont_def}.\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   915
  assumes infsum: \<open>(g has_sum x) S\<close>
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   916
  shows \<open>((f \<circ> g) has_sum (f x)) S\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   917
  using assms
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   918
  by (intro has_sum_comm_additive_general has_sum_infsum) (auto simp: isCont_def additive.sum) 
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   919
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   920
lemma summable_on_comm_additive:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   921
  fixes f :: \<open>'b :: {ab_group_add,t2_space} \<Rightarrow> 'c :: {ab_group_add,topological_space}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   922
  assumes \<open>additive f\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   923
  assumes \<open>isCont f (infsum g S)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   924
  assumes \<open>g summable_on S\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   925
  shows \<open>(f \<circ> g) summable_on S\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   926
  by (meson assms summable_on_def has_sum_comm_additive has_sum_infsum isContD)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   927
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   928
lemma infsum_comm_additive:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   929
  fixes f :: \<open>'b :: {ab_group_add,t2_space} \<Rightarrow> 'c :: {ab_group_add,t2_space}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   930
  assumes \<open>additive f\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   931
  assumes \<open>isCont f (infsum g S)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   932
  assumes \<open>g summable_on S\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   933
  shows \<open>infsum (f \<circ> g) S = f (infsum g S)\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   934
  by (rule infsum_comm_additive_general; auto simp: assms additive.sum)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   935
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   936
lemma nonneg_bdd_above_has_sum:
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   937
  fixes f :: \<open>'a \<Rightarrow> 'b :: {conditionally_complete_linorder, ordered_comm_monoid_add, linorder_topology}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   938
  assumes \<open>\<And>x. x\<in>A \<Longrightarrow> f x \<ge> 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   939
  assumes \<open>bdd_above (sum f ` {F. F\<subseteq>A \<and> finite F})\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   940
  shows \<open>(f has_sum (SUP F\<in>{F. finite F \<and> F\<subseteq>A}. sum f F)) A\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   941
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   942
  have \<open>(sum f \<longlongrightarrow> (SUP F\<in>{F. finite F \<and> F\<subseteq>A}. sum f F)) (finite_subsets_at_top A)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   943
  proof (rule order_tendstoI)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   944
    fix a assume \<open>a < (SUP F\<in>{F. finite F \<and> F\<subseteq>A}. sum f F)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   945
    then obtain F where \<open>a < sum f F\<close> and \<open>finite F\<close> and \<open>F \<subseteq> A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   946
      by (metis (mono_tags, lifting) Collect_cong Collect_empty_eq assms(2) empty_subsetI finite.emptyI less_cSUP_iff mem_Collect_eq)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   947
    have "\<And>Y. \<lbrakk>finite Y; F \<subseteq> Y; Y \<subseteq> A\<rbrakk> \<Longrightarrow> a < sum f Y"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   948
      by (meson DiffE \<open>a < sum f F\<close> assms(1) less_le_trans subset_iff sum_mono2)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   949
    then show \<open>\<forall>\<^sub>F x in finite_subsets_at_top A. a < sum f x\<close>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   950
      by (metis \<open>F \<subseteq> A\<close> \<open>finite F\<close> eventually_finite_subsets_at_top)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   951
  next
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   952
    fix a assume *: \<open>(SUP F\<in>{F. finite F \<and> F\<subseteq>A}. sum f F) < a\<close>
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
   953
    have "sum f F \<le> (SUP F\<in>{F. finite F \<and> F\<subseteq>A}. sum f F)" if \<open>F\<subseteq>A\<close> and \<open>finite F\<close> for F
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   954
        by (rule cSUP_upper) (use that assms(2) in \<open>auto simp: conj_commute\<close>)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   955
    then show \<open>\<forall>\<^sub>F x in finite_subsets_at_top A. sum f x < a\<close>
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
   956
      by (metis (no_types, lifting) "*" eventually_finite_subsets_at_top_weakI order_le_less_trans)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   957
  qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   958
  then show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   959
    using has_sum_def by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   960
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   961
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   962
lemma nonneg_bdd_above_summable_on:
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   963
  fixes f :: \<open>'a \<Rightarrow> 'b :: {conditionally_complete_linorder, ordered_comm_monoid_add, linorder_topology}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   964
  assumes \<open>\<And>x. x\<in>A \<Longrightarrow> f x \<ge> 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   965
  assumes \<open>bdd_above (sum f ` {F. F\<subseteq>A \<and> finite F})\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   966
  shows \<open>f summable_on A\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   967
  using assms summable_on_def nonneg_bdd_above_has_sum by blast
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   968
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   969
lemma nonneg_bdd_above_infsum:
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   970
  fixes f :: \<open>'a \<Rightarrow> 'b :: {conditionally_complete_linorder, ordered_comm_monoid_add, linorder_topology}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   971
  assumes \<open>\<And>x. x\<in>A \<Longrightarrow> f x \<ge> 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   972
  assumes \<open>bdd_above (sum f ` {F. F\<subseteq>A \<and> finite F})\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   973
  shows \<open>infsum f A = (SUP F\<in>{F. finite F \<and> F\<subseteq>A}. sum f F)\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   974
  using assms by (auto intro!: infsumI nonneg_bdd_above_has_sum)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   975
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   976
lemma nonneg_has_sum_complete:
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   977
  fixes f :: \<open>'a \<Rightarrow> 'b :: {complete_linorder, ordered_comm_monoid_add, linorder_topology}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   978
  assumes \<open>\<And>x. x\<in>A \<Longrightarrow> f x \<ge> 0\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   979
  shows \<open>(f has_sum (SUP F\<in>{F. finite F \<and> F\<subseteq>A}. sum f F)) A\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   980
  using assms nonneg_bdd_above_has_sum by blast
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   981
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   982
lemma nonneg_summable_on_complete:
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   983
  fixes f :: \<open>'a \<Rightarrow> 'b :: {complete_linorder, ordered_comm_monoid_add, linorder_topology}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   984
  assumes \<open>\<And>x. x\<in>A \<Longrightarrow> f x \<ge> 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   985
  shows \<open>f summable_on A\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   986
  using assms nonneg_bdd_above_summable_on by blast
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   987
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   988
lemma nonneg_infsum_complete:
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   989
  fixes f :: \<open>'a \<Rightarrow> 'b :: {complete_linorder, ordered_comm_monoid_add, linorder_topology}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   990
  assumes \<open>\<And>x. x\<in>A \<Longrightarrow> f x \<ge> 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   991
  shows \<open>infsum f A = (SUP F\<in>{F. finite F \<and> F\<subseteq>A}. sum f F)\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
   992
  using assms nonneg_bdd_above_infsum by blast
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   993
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   994
lemma has_sum_nonneg:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   995
  fixes f :: "'a \<Rightarrow> 'b::{ordered_comm_monoid_add,linorder_topology}"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
   996
  assumes "(f has_sum a) M"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   997
    and "\<And>x. x \<in> M \<Longrightarrow> 0 \<le> f x"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
   998
  shows "a \<ge> 0"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
   999
  by (metis (no_types, lifting) DiffD1 assms empty_iff has_sum_0 has_sum_mono_neutral order_refl)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1000
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1001
lemma infsum_nonneg:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1002
  fixes f :: "'a \<Rightarrow> 'b::{ordered_comm_monoid_add,linorder_topology}"
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1003
  assumes "\<And>x. x \<in> M \<Longrightarrow> 0 \<le> f x"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1004
  shows "infsum f M \<ge> 0" (is "?lhs \<ge> _")
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1005
  by (metis assms has_sum_infsum has_sum_nonneg infsum_not_exists linorder_linear)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1006
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1007
lemma has_sum_mono2:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1008
  fixes f :: "'a \<Rightarrow> 'b::{topological_ab_group_add, ordered_comm_monoid_add,linorder_topology}"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1009
  assumes "(f has_sum S) A" "(f has_sum S') B" "A \<subseteq> B"
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1010
  assumes "\<And>x. x \<in> B - A \<Longrightarrow> f x \<ge> 0"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1011
  shows   "S \<le> S'"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1012
  by (metis add_0 add_right_mono assms diff_add_cancel has_sum_Diff has_sum_nonneg)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1013
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1014
lemma infsum_mono2:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1015
  fixes f :: "'a \<Rightarrow> 'b::{topological_ab_group_add, ordered_comm_monoid_add,linorder_topology}"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1016
  assumes "f summable_on A" "f summable_on B" "A \<subseteq> B"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1017
  assumes "\<And>x. x \<in> B - A \<Longrightarrow> f x \<ge> 0"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1018
  shows   "infsum f A \<le> infsum f B"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1019
  by (rule has_sum_mono2[OF has_sum_infsum has_sum_infsum]) (use assms in auto)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1020
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1021
lemma finite_sum_le_has_sum:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1022
  fixes f :: "'a \<Rightarrow> 'b::{topological_ab_group_add, ordered_comm_monoid_add,linorder_topology}"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1023
  assumes "(f has_sum S) A" "finite B" "B \<subseteq> A"
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1024
  assumes "\<And>x. x \<in> A - B \<Longrightarrow> f x \<ge> 0"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1025
  shows   "sum f B \<le> S"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1026
  by (meson assms has_sum_finite has_sum_mono2)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1027
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1028
lemma finite_sum_le_infsum:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1029
  fixes f :: "'a \<Rightarrow> 'b::{topological_ab_group_add, ordered_comm_monoid_add,linorder_topology}"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1030
  assumes "f summable_on A" "finite B" "B \<subseteq> A"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1031
  assumes "\<And>x. x \<in> A - B \<Longrightarrow> f x \<ge> 0"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1032
  shows   "sum f B \<le> infsum f A"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1033
  by (rule finite_sum_le_has_sum[OF has_sum_infsum]) (use assms in auto)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1034
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1035
lemma has_sum_reindex:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1036
  assumes \<open>inj_on h A\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1037
  shows \<open>(g has_sum x) (h ` A) \<longleftrightarrow> ((g \<circ> h) has_sum x) A\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1038
proof -
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1039
  have \<open>(g has_sum x) (h ` A) \<longleftrightarrow> (sum g \<longlongrightarrow> x) (finite_subsets_at_top (h ` A))\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1040
    by (simp add: has_sum_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1041
  also have \<open>\<dots> \<longleftrightarrow> ((\<lambda>F. sum g (h ` F)) \<longlongrightarrow> x) (finite_subsets_at_top A)\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1042
    by (metis assms filterlim_filtermap filtermap_image_finite_subsets_at_top)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1043
  also have \<open>\<dots> \<longleftrightarrow> (sum (g \<circ> h) \<longlongrightarrow> x) (finite_subsets_at_top A)\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1044
  proof (intro tendsto_cong eventually_finite_subsets_at_top_weakI sum.reindex)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1045
    show "\<And>X. \<lbrakk>finite X; X \<subseteq> A\<rbrakk> \<Longrightarrow> inj_on h X"
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1046
      using assms subset_inj_on by blast
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1047
  qed
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1048
  also have \<open>\<dots> \<longleftrightarrow> ((g \<circ> h) has_sum x) A\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1049
    by (simp add: has_sum_def)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1050
  finally show ?thesis .
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1051
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1052
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1053
lemma summable_on_reindex:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1054
  assumes \<open>inj_on h A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1055
  shows \<open>g summable_on (h ` A) \<longleftrightarrow> (g \<circ> h) summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1056
  by (simp add: assms summable_on_def has_sum_reindex)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1057
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1058
lemma infsum_reindex:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1059
  assumes \<open>inj_on h A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1060
  shows \<open>infsum g (h ` A) = infsum (g \<circ> h) A\<close>
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1061
  by (metis assms has_sum_infsum has_sum_reindex infsumI infsum_def)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1062
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1063
lemma summable_on_reindex_bij_betw:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1064
  assumes "bij_betw g A B"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1065
  shows   "(\<lambda>x. f (g x)) summable_on A \<longleftrightarrow> f summable_on B"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1066
  by (smt (verit) assms bij_betw_def o_apply summable_on_cong summable_on_reindex) 
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1067
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1068
lemma infsum_reindex_bij_betw:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1069
  assumes "bij_betw g A B"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1070
  shows   "infsum (\<lambda>x. f (g x)) A = infsum f B"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1071
  by (metis (mono_tags, lifting) assms bij_betw_def infsum_cong infsum_reindex o_def)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1072
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1073
lemma sum_uniformity:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1074
  assumes plus_cont: \<open>uniformly_continuous_on UNIV (\<lambda>(x::'b::{uniform_space,comm_monoid_add},y). x+y)\<close>
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1075
  assumes EE: \<open>eventually E uniformity\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1076
  obtains D where \<open>eventually D uniformity\<close> 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1077
    and \<open>\<And>M::'a set. \<And>f f' :: 'a \<Rightarrow> 'b. card M \<le> n \<and> (\<forall>m\<in>M. D (f m, f' m)) \<Longrightarrow> E (sum f M, sum f' M)\<close>
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1078
proof (atomize_elim, insert EE, induction n arbitrary: E rule:nat_induct)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1079
  case 0
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1080
  then show ?case
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1081
    by (metis card_eq_0_iff equals0D le_zero_eq sum.infinite sum.not_neutral_contains_not_neutral uniformity_refl)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1082
next
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1083
  case (Suc n)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1084
  from plus_cont[unfolded uniformly_continuous_on_uniformity filterlim_def le_filter_def, rule_format, OF Suc.prems]
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1085
  obtain D1 D2 where \<open>eventually D1 uniformity\<close> and \<open>eventually D2 uniformity\<close> 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1086
    and D1D2E: \<open>D1 (x, y) \<Longrightarrow> D2 (x', y') \<Longrightarrow> E (x + x', y + y')\<close> for x y x' y'
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1087
    apply atomize_elim
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1088
    by (auto simp: eventually_prod_filter case_prod_beta uniformity_prod_def eventually_filtermap)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1089
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1090
  from Suc.IH[OF \<open>eventually D2 uniformity\<close>]
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1091
  obtain D3 where \<open>eventually D3 uniformity\<close> and D3: \<open>card M \<le> n \<Longrightarrow> (\<forall>m\<in>M. D3 (f m, f' m)) \<Longrightarrow> D2 (sum f M, sum f' M)\<close> 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1092
    for M :: \<open>'a set\<close> and f f'
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1093
    by metis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1094
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1095
  define D where \<open>D x \<equiv> D1 x \<and> D3 x\<close> for x
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1096
  have \<open>eventually D uniformity\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1097
    using D_def \<open>eventually D1 uniformity\<close> \<open>eventually D3 uniformity\<close> eventually_elim2 by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1098
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1099
  have \<open>E (sum f M, sum f' M)\<close> 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1100
    if \<open>card M \<le> Suc n\<close> and DM: \<open>\<forall>m\<in>M. D (f m, f' m)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1101
    for M :: \<open>'a set\<close> and f f'
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1102
  proof (cases \<open>card M = 0\<close>)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1103
    case True
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1104
    then show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1105
      by (metis Suc.prems card_eq_0_iff sum.empty sum.infinite uniformity_refl) 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1106
  next
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1107
    case False
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1108
    with \<open>card M \<le> Suc n\<close> obtain N x where \<open>card N \<le> n\<close> and \<open>x \<notin> N\<close> and \<open>M = insert x N\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1109
      by (metis card_Suc_eq less_Suc_eq_0_disj less_Suc_eq_le)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1110
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1111
    from DM have \<open>\<And>m. m\<in>N \<Longrightarrow> D (f m, f' m)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1112
      using \<open>M = insert x N\<close> by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1113
    with D3[OF \<open>card N \<le> n\<close>]
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1114
    have D2_N: \<open>D2 (sum f N, sum f' N)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1115
      using D_def by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1116
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1117
    from DM 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1118
    have \<open>D (f x, f' x)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1119
      using \<open>M = insert x N\<close> by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1120
    then have \<open>D1 (f x, f' x)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1121
      by (simp add: D_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1122
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1123
    with D2_N
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1124
    have \<open>E (f x + sum f N, f' x + sum f' N)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1125
      using D1D2E by presburger
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1126
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1127
    then show \<open>E (sum f M, sum f' M)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1128
      by (metis False \<open>M = insert x N\<close> \<open>x \<notin> N\<close> card.infinite finite_insert sum.insert)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1129
  qed
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1130
  with \<open>eventually D uniformity\<close> show ?case 
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1131
    by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1132
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1133
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1134
lemma has_sum_Sigma:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1135
  fixes A :: "'a set" and B :: "'a \<Rightarrow> 'b set"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1136
    and f :: \<open>'a \<times> 'b \<Rightarrow> 'c::{comm_monoid_add,uniform_space}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1137
  assumes plus_cont: \<open>uniformly_continuous_on UNIV (\<lambda>(x::'c,y). x+y)\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1138
  assumes summableAB: "(f has_sum a) (Sigma A B)"
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1139
  assumes summableB: \<open>\<And>x. x\<in>A \<Longrightarrow> ((\<lambda>y. f (x, y)) has_sum b x) (B x)\<close>
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1140
  shows "(b has_sum a) A"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1141
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1142
  define F FB FA where \<open>F = finite_subsets_at_top (Sigma A B)\<close> and \<open>FB x = finite_subsets_at_top (B x)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1143
    and \<open>FA = finite_subsets_at_top A\<close> for x
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1144
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1145
  from summableB
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1146
  have sum_b: \<open>(sum (\<lambda>y. f (x, y)) \<longlongrightarrow> b x) (FB x)\<close> if \<open>x \<in> A\<close> for x
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1147
    using FB_def[abs_def] has_sum_def that by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1148
  from summableAB
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1149
  have sum_S: \<open>(sum f \<longlongrightarrow> a) F\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1150
    using F_def has_sum_def by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1151
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1152
  have finite_proj: \<open>finite {b| b. (a,b) \<in> H}\<close> if \<open>finite H\<close> for H :: \<open>('a\<times>'b) set\<close> and a
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1153
    by (metis (no_types, lifting) finite_imageI finite_subset image_eqI mem_Collect_eq snd_conv subsetI that)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1154
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1155
  have \<open>(sum b \<longlongrightarrow> a) FA\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1156
  proof (rule tendsto_iff_uniformity[THEN iffD2, rule_format])
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1157
    fix E :: \<open>('c \<times> 'c) \<Rightarrow> bool\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1158
    assume \<open>eventually E uniformity\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1159
    then obtain D where D_uni: \<open>eventually D uniformity\<close> and DDE': \<open>\<And>x y z. D (x, y) \<Longrightarrow> D (y, z) \<Longrightarrow> E (x, z)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1160
      by (metis (no_types, lifting) \<open>eventually E uniformity\<close> uniformity_transE)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1161
    from sum_S obtain G where \<open>finite G\<close> and \<open>G \<subseteq> Sigma A B\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1162
      and G_sum: \<open>G \<subseteq> H \<Longrightarrow> H \<subseteq> Sigma A B \<Longrightarrow> finite H \<Longrightarrow> D (sum f H, a)\<close> for H
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1163
      unfolding tendsto_iff_uniformity
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1164
      by (metis (mono_tags, lifting) D_uni F_def eventually_finite_subsets_at_top)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1165
    have \<open>finite (fst ` G)\<close> and \<open>fst ` G \<subseteq> A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1166
      using \<open>finite G\<close> \<open>G \<subseteq> Sigma A B\<close> by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1167
    thm uniformity_prod_def
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1168
    define Ga where \<open>Ga a = {b. (a,b) \<in> G}\<close> for a
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1169
    have Ga_fin: \<open>finite (Ga a)\<close> and Ga_B: \<open>Ga a \<subseteq> B a\<close> for a
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1170
      using \<open>finite G\<close> \<open>G \<subseteq> Sigma A B\<close> finite_proj by (auto simp: Ga_def finite_proj)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1171
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1172
    have \<open>E (sum b M, a)\<close> if \<open>M \<supseteq> fst ` G\<close> and \<open>finite M\<close> and \<open>M \<subseteq> A\<close> for M
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1173
    proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1174
      define FMB where \<open>FMB = finite_subsets_at_top (Sigma M B)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1175
      have \<open>eventually (\<lambda>H. D (\<Sum>a\<in>M. b a, \<Sum>(a,b)\<in>H. f (a,b))) FMB\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1176
      proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1177
        obtain D' where D'_uni: \<open>eventually D' uniformity\<close> 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1178
          and \<open>card M' \<le> card M \<and> (\<forall>m\<in>M'. D' (g m, g' m)) \<Longrightarrow> D (sum g M', sum g' M')\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1179
        for M' :: \<open>'a set\<close> and g g'
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1180
          using sum_uniformity[OF plus_cont \<open>eventually D uniformity\<close>] by blast
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1181
        then have D'_sum_D: \<open>(\<forall>m\<in>M. D' (g m, g' m)) \<Longrightarrow> D (sum g M, sum g' M)\<close> for g g'
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1182
          by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1183
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1184
        obtain Ha where \<open>Ha a \<supseteq> Ga a\<close> and Ha_fin: \<open>finite (Ha a)\<close> and Ha_B: \<open>Ha a \<subseteq> B a\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1185
          and D'_sum_Ha: \<open>Ha a \<subseteq> L \<Longrightarrow> L \<subseteq> B a \<Longrightarrow> finite L \<Longrightarrow> D' (b a, sum (\<lambda>b. f (a,b)) L)\<close> if \<open>a \<in> A\<close> for a L
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1186
        proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1187
          from sum_b[unfolded tendsto_iff_uniformity, rule_format, OF _ D'_uni[THEN uniformity_sym]]
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1188
          obtain Ha0 where \<open>finite (Ha0 a)\<close> and \<open>Ha0 a \<subseteq> B a\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1189
            and \<open>Ha0 a \<subseteq> L \<Longrightarrow> L \<subseteq> B a \<Longrightarrow> finite L \<Longrightarrow> D' (b a, sum (\<lambda>b. f (a,b)) L)\<close> if \<open>a \<in> A\<close> for a L
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1190
            unfolding FB_def eventually_finite_subsets_at_top unfolding prod.case by metis
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1191
          moreover define Ha where \<open>Ha a = Ha0 a \<union> Ga a\<close> for a
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1192
          ultimately show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1193
            using that[where Ha=Ha]
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1194
            using Ga_fin Ga_B by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1195
        qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1196
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1197
        have \<open>D (\<Sum>a\<in>M. b a, \<Sum>(a,b)\<in>H. f (a,b))\<close> if \<open>finite H\<close> and \<open>H \<subseteq> Sigma M B\<close> and \<open>H \<supseteq> Sigma M Ha\<close> for H
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1198
        proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1199
          define Ha' where \<open>Ha' a = {b| b. (a,b) \<in> H}\<close> for a
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1200
          have [simp]: \<open>finite (Ha' a)\<close> and [simp]: \<open>Ha' a \<supseteq> Ha a\<close> and [simp]: \<open>Ha' a \<subseteq> B a\<close> if \<open>a \<in> M\<close> for a
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1201
            unfolding Ha'_def using \<open>finite H\<close> \<open>H \<subseteq> Sigma M B\<close> \<open>Sigma M Ha \<subseteq> H\<close> that finite_proj by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1202
          have \<open>Sigma M Ha' = H\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1203
            using that by (auto simp: Ha'_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1204
          then have *: \<open>(\<Sum>(a,b)\<in>H. f (a,b)) = (\<Sum>a\<in>M. \<Sum>b\<in>Ha' a. f (a,b))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1205
            by (simp add: \<open>finite M\<close> sum.Sigma)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1206
          have \<open>D' (b a, sum (\<lambda>b. f (a,b)) (Ha' a))\<close> if \<open>a \<in> M\<close> for a
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1207
            using D'_sum_Ha \<open>M \<subseteq> A\<close> that by auto
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1208
          then have \<open>D (\<Sum>a\<in>M. b a, \<Sum>a\<in>M. sum (\<lambda>b. f (a,b)) (Ha' a))\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1209
            by (rule_tac D'_sum_D, auto)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1210
          with * show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1211
            by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1212
        qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1213
        moreover have \<open>Sigma M Ha \<subseteq> Sigma M B\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1214
          using Ha_B \<open>M \<subseteq> A\<close> by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1215
        ultimately show ?thesis
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1216
          unfolding FMB_def eventually_finite_subsets_at_top
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1217
          by (metis (no_types, lifting) Ha_fin finite_SigmaI subsetD that(2) that(3))
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1218
      qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1219
      moreover have \<open>eventually (\<lambda>H. D (\<Sum>(a,b)\<in>H. f (a,b), a)) FMB\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1220
        unfolding FMB_def eventually_finite_subsets_at_top
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1221
      proof (rule exI[of _ G], safe)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1222
        fix Y assume Y: "finite Y" "G \<subseteq> Y" "Y \<subseteq> Sigma M B"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1223
        thus "D (\<Sum>(a,b)\<in>Y. f (a, b), a)"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1224
          using G_sum[of Y] Y using that(3) by fastforce
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1225
      qed (use \<open>finite G\<close> \<open>G \<subseteq> Sigma A B\<close> that in auto)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1226
      ultimately have \<open>\<forall>\<^sub>F x in FMB. E (sum b M, a)\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1227
        by eventually_elim (use DDE' in auto)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1228
      then show \<open>E (sum b M, a)\<close>
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1229
        using FMB_def by force
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1230
    qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1231
    then show \<open>\<forall>\<^sub>F x in FA. E (sum b x, a)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1232
      using \<open>finite (fst ` G)\<close> and \<open>fst ` G \<subseteq> A\<close>
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1233
      by (metis (mono_tags, lifting) FA_def eventually_finite_subsets_at_top)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1234
  qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1235
  then show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1236
    by (simp add: FA_def has_sum_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1237
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1238
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1239
lemma summable_on_Sigma:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1240
  fixes A :: "'a set" and B :: "'a \<Rightarrow> 'b set"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1241
    and f :: \<open>'a \<Rightarrow> 'b \<Rightarrow> 'c::{comm_monoid_add, t2_space, uniform_space}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1242
  assumes plus_cont: \<open>uniformly_continuous_on UNIV (\<lambda>(x::'c,y). x+y)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1243
  assumes summableAB: "(\<lambda>(x,y). f x y) summable_on (Sigma A B)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1244
  assumes summableB: \<open>\<And>x. x\<in>A \<Longrightarrow> (f x) summable_on (B x)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1245
  shows \<open>(\<lambda>x. infsum (f x) (B x)) summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1246
proof -
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1247
  from summableAB obtain a where a: \<open>((\<lambda>(x,y). f x y) has_sum a) (Sigma A B)\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1248
    using has_sum_infsum by blast
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1249
  from summableB have b: \<open>\<And>x. x\<in>A \<Longrightarrow> (f x has_sum infsum (f x) (B x)) (B x)\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1250
    by (auto intro!: has_sum_infsum)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1251
  show ?thesis
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1252
    using plus_cont a b
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1253
    by (smt (verit) has_sum_Sigma[where f=\<open>\<lambda>(x,y). f x y\<close>] has_sum_cong old.prod.case summable_on_def) 
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1254
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1255
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1256
lemma infsum_Sigma:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1257
  fixes A :: "'a set" and B :: "'a \<Rightarrow> 'b set"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1258
    and f :: \<open>'a \<times> 'b \<Rightarrow> 'c::{comm_monoid_add, t2_space, uniform_space}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1259
  assumes plus_cont: \<open>uniformly_continuous_on UNIV (\<lambda>(x::'c,y). x+y)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1260
  assumes summableAB: "f summable_on (Sigma A B)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1261
  assumes summableB: \<open>\<And>x. x\<in>A \<Longrightarrow> (\<lambda>y. f (x, y)) summable_on (B x)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1262
  shows "infsum f (Sigma A B) = infsum (\<lambda>x. infsum (\<lambda>y. f (x, y)) (B x)) A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1263
proof -
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1264
  from summableAB have a: \<open>(f has_sum infsum f (Sigma A B)) (Sigma A B)\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1265
    using has_sum_infsum by blast
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1266
  from summableB have b: \<open>\<And>x. x\<in>A \<Longrightarrow> ((\<lambda>y. f (x, y)) has_sum infsum (\<lambda>y. f (x, y)) (B x)) (B x)\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1267
    by (auto intro!: has_sum_infsum)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1268
  show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1269
    using plus_cont a b by (auto intro: infsumI[symmetric] has_sum_Sigma simp: summable_on_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1270
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1271
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1272
lemma infsum_Sigma':
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1273
  fixes A :: "'a set" and B :: "'a \<Rightarrow> 'b set"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1274
    and f :: \<open>'a \<Rightarrow> 'b \<Rightarrow> 'c::{comm_monoid_add, t2_space, uniform_space}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1275
  assumes plus_cont: \<open>uniformly_continuous_on UNIV (\<lambda>(x::'c,y). x+y)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1276
  assumes summableAB: "(\<lambda>(x,y). f x y) summable_on (Sigma A B)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1277
  assumes summableB: \<open>\<And>x. x\<in>A \<Longrightarrow> (f x) summable_on (B x)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1278
  shows \<open>infsum (\<lambda>x. infsum (f x) (B x)) A = infsum (\<lambda>(x,y). f x y) (Sigma A B)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1279
  using infsum_Sigma[of \<open>\<lambda>(x,y). f x y\<close> A B]
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1280
  using assms by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1281
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1282
text \<open>A special case of @{thm [source] infsum_Sigma} etc. for Banach spaces. It has less premises.\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1283
lemma
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1284
  fixes A :: "'a set" and B :: "'a \<Rightarrow> 'b set"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1285
    and f :: \<open>'a \<Rightarrow> 'b \<Rightarrow> 'c::banach\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1286
  assumes [simp]: "(\<lambda>(x,y). f x y) summable_on (Sigma A B)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1287
  shows infsum_Sigma'_banach: \<open>infsum (\<lambda>x. infsum (f x) (B x)) A = infsum (\<lambda>(x,y). f x y) (Sigma A B)\<close> (is ?thesis1)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1288
    and summable_on_Sigma_banach: \<open>(\<lambda>x. infsum (f x) (B x)) summable_on A\<close> (is ?thesis2)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1289
proof -
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1290
  have fsum: \<open>(f x) summable_on (B x)\<close> if \<open>x \<in> A\<close> for x
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1291
  proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1292
    from assms
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1293
    have \<open>(\<lambda>(x,y). f x y) summable_on (Pair x ` B x)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1294
      by (meson image_subset_iff summable_on_subset_banach mem_Sigma_iff that)
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1295
    then have \<open>((\<lambda>(x,y). f x y) \<circ> Pair x) summable_on (B x)\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1296
      by (metis summable_on_reindex inj_on_def prod.inject)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1297
    then show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1298
      by (auto simp: o_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1299
  qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1300
  show ?thesis1
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1301
    using fsum assms infsum_Sigma' isUCont_plus by blast
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1302
  show ?thesis2
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1303
    using fsum assms isUCont_plus summable_on_Sigma by blast
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1304
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1305
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1306
lemma infsum_Sigma_banach:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1307
  fixes A :: "'a set" and B :: "'a \<Rightarrow> 'b set"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1308
    and f :: \<open>'a \<times> 'b \<Rightarrow> 'c::banach\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1309
  assumes [simp]: "f summable_on (Sigma A B)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1310
  shows \<open>infsum (\<lambda>x. infsum (\<lambda>y. f (x,y)) (B x)) A = infsum f (Sigma A B)\<close>
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1311
  using assms by (simp add: infsum_Sigma'_banach)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1312
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1313
lemma infsum_swap:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1314
  fixes A :: "'a set" and B :: "'b set"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1315
  fixes f :: "'a \<Rightarrow> 'b \<Rightarrow> 'c::{comm_monoid_add,t2_space,uniform_space}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1316
  assumes plus_cont: \<open>uniformly_continuous_on UNIV (\<lambda>(x::'c,y). x+y)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1317
  assumes \<open>(\<lambda>(x, y). f x y) summable_on (A \<times> B)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1318
  assumes \<open>\<And>a. a\<in>A \<Longrightarrow> (f a) summable_on B\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1319
  assumes \<open>\<And>b. b\<in>B \<Longrightarrow> (\<lambda>a. f a b) summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1320
  shows \<open>infsum (\<lambda>x. infsum (\<lambda>y. f x y) B) A = infsum (\<lambda>y. infsum (\<lambda>x. f x y) A) B\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1321
proof -
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1322
  have "(\<lambda>(x, y). f y x) \<circ> prod.swap summable_on A \<times> B"
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1323
    by (simp add: assms(2) summable_on_cong)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1324
  then have fyx: \<open>(\<lambda>(x, y). f y x) summable_on (B \<times> A)\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1325
    by (metis has_sum_reindex infsum_reindex inj_swap product_swap summable_iff_has_sum_infsum)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1326
  have \<open>infsum (\<lambda>x. infsum (\<lambda>y. f x y) B) A = infsum (\<lambda>(x,y). f x y) (A \<times> B)\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1327
    using assms infsum_Sigma' by blast
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1328
  also have \<open>\<dots> = infsum (\<lambda>(x,y). f y x) (B \<times> A)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1329
    apply (subst product_swap[symmetric])
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1330
    apply (subst infsum_reindex)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1331
    using assms by (auto simp: o_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1332
  also have \<open>\<dots> = infsum (\<lambda>y. infsum (\<lambda>x. f x y) A) B\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1333
    by (smt (verit) fyx assms(1) assms(4) infsum_Sigma' infsum_cong)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1334
  finally show ?thesis .
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1335
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1336
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1337
lemma infsum_swap_banach:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1338
  fixes A :: "'a set" and B :: "'b set"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1339
  fixes f :: "'a \<Rightarrow> 'b \<Rightarrow> 'c::banach"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1340
  assumes \<open>(\<lambda>(x, y). f x y) summable_on (A \<times> B)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1341
  shows "infsum (\<lambda>x. infsum (\<lambda>y. f x y) B) A = infsum (\<lambda>y. infsum (\<lambda>x. f x y) A) B"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1342
proof -
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1343
  have \<section>: \<open>(\<lambda>(x, y). f y x) summable_on (B \<times> A)\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1344
    by (metis (mono_tags, lifting) assms case_swap inj_swap o_apply product_swap summable_on_cong summable_on_reindex)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1345
  have \<open>infsum (\<lambda>x. infsum (\<lambda>y. f x y) B) A = infsum (\<lambda>(x,y). f x y) (A \<times> B)\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1346
    using assms infsum_Sigma'_banach by blast
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1347
  also have \<open>\<dots> = infsum (\<lambda>(x,y). f y x) (B \<times> A)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1348
    apply (subst product_swap[symmetric])
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1349
    apply (subst infsum_reindex)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1350
    using assms by (auto simp: o_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1351
  also have \<open>\<dots> = infsum (\<lambda>y. infsum (\<lambda>x. f x y) A) B\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1352
    by (metis (mono_tags, lifting) \<section> infsum_Sigma'_banach infsum_cong)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1353
  finally show ?thesis .
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1354
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1355
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1356
lemma nonneg_infsum_le_0D:
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1357
  fixes f :: "'a \<Rightarrow> 'b::{topological_ab_group_add,ordered_ab_group_add,linorder_topology}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1358
  assumes "infsum f A \<le> 0"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1359
    and abs_sum: "f summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1360
    and nneg: "\<And>x. x \<in> A \<Longrightarrow> f x \<ge> 0"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1361
    and "x \<in> A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1362
  shows "f x = 0"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1363
proof (rule ccontr)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1364
  assume \<open>f x \<noteq> 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1365
  have ex: \<open>f summable_on (A-{x})\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1366
    by (rule summable_on_cofin_subset) (use assms in auto)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1367
  have pos: \<open>infsum f (A - {x}) \<ge> 0\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1368
    by (rule infsum_nonneg) (use nneg in auto)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1369
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1370
  have [trans]: \<open>x \<ge> y \<Longrightarrow> y > z \<Longrightarrow> x > z\<close> for x y z :: 'b by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1371
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1372
  have \<open>infsum f A = infsum f (A-{x}) + infsum f {x}\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1373
    by (subst infsum_Un_disjoint[symmetric]) (use assms ex in \<open>auto simp: insert_absorb\<close>)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1374
  also have \<open>\<dots> \<ge> infsum f {x}\<close> (is \<open>_ \<ge> \<dots>\<close>)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1375
    using pos by (rule add_increasing) simp
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1376
  also have \<open>\<dots> = f x\<close> (is \<open>_ = \<dots>\<close>)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1377
    by (subst infsum_finite) auto
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1378
  also have \<open>\<dots> > 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1379
    using \<open>f x \<noteq> 0\<close> assms(4) nneg by fastforce
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1380
  finally show False
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1381
    using assms by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1382
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1383
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1384
lemma nonneg_has_sum_le_0D:
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1385
  fixes f :: "'a \<Rightarrow> 'b::{topological_ab_group_add,ordered_ab_group_add,linorder_topology}"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1386
  assumes "(f has_sum a) A" \<open>a \<le> 0\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1387
    and "\<And>x. x \<in> A \<Longrightarrow> f x \<ge> 0"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1388
    and "x \<in> A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1389
  shows "f x = 0"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1390
  by (metis assms infsumI nonneg_infsum_le_0D summable_on_def)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1391
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1392
lemma has_sum_cmult_left:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1393
  fixes f :: "'a \<Rightarrow> 'b :: {topological_semigroup_mult, semiring_0}"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1394
  assumes \<open>(f has_sum a) A\<close>
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1395
  shows "((\<lambda>x. f x * c) has_sum (a * c)) A"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1396
  using assms tendsto_mult_right 
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1397
  by (force simp add: has_sum_def sum_distrib_right)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1398
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1399
lemma infsum_cmult_left:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1400
  fixes f :: "'a \<Rightarrow> 'b :: {t2_space, topological_semigroup_mult, semiring_0}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1401
  assumes \<open>c \<noteq> 0 \<Longrightarrow> f summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1402
  shows "infsum (\<lambda>x. f x * c) A = infsum f A * c"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1403
  using assms has_sum_cmult_left infsumI summable_iff_has_sum_infsum by fastforce
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1404
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1405
lemma summable_on_cmult_left:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1406
  fixes f :: "'a \<Rightarrow> 'b :: {t2_space, topological_semigroup_mult, semiring_0}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1407
  assumes \<open>f summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1408
  shows "(\<lambda>x. f x * c) summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1409
  using assms summable_on_def has_sum_cmult_left by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1410
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1411
lemma has_sum_cmult_right:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1412
  fixes f :: "'a \<Rightarrow> 'b :: {topological_semigroup_mult, semiring_0}"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1413
  assumes \<open>(f has_sum a) A\<close>
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1414
  shows "((\<lambda>x. c * f x) has_sum (c * a)) A"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1415
  using assms tendsto_mult_left 
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1416
  by (force simp add: has_sum_def sum_distrib_left)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1417
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1418
lemma infsum_cmult_right:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1419
  fixes f :: "'a \<Rightarrow> 'b :: {t2_space, topological_semigroup_mult, semiring_0}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1420
  assumes \<open>c \<noteq> 0 \<Longrightarrow> f summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1421
  shows \<open>infsum (\<lambda>x. c * f x) A = c * infsum f A\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1422
  using assms has_sum_cmult_right infsumI summable_iff_has_sum_infsum by fastforce
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1423
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1424
lemma summable_on_cmult_right:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1425
  fixes f :: "'a \<Rightarrow> 'b :: {t2_space, topological_semigroup_mult, semiring_0}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1426
  assumes \<open>f summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1427
  shows "(\<lambda>x. c * f x) summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1428
  using assms summable_on_def has_sum_cmult_right by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1429
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1430
lemma summable_on_cmult_left':
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1431
  fixes f :: "'a \<Rightarrow> 'b :: {t2_space, topological_semigroup_mult, division_ring}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1432
  assumes \<open>c \<noteq> 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1433
  shows "(\<lambda>x. f x * c) summable_on A \<longleftrightarrow> f summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1434
proof
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1435
  assume \<open>f summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1436
  then show \<open>(\<lambda>x. f x * c) summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1437
    by (rule summable_on_cmult_left)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1438
next
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1439
  assume \<open>(\<lambda>x. f x * c) summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1440
  then have \<open>(\<lambda>x. f x * c * inverse c) summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1441
    by (rule summable_on_cmult_left)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1442
  then show \<open>f summable_on A\<close>
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1443
    by (smt (verit, del_insts) assms divide_inverse nonzero_divide_eq_eq summable_on_cong)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1444
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1445
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1446
lemma summable_on_cmult_right':
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1447
  fixes f :: "'a \<Rightarrow> 'b :: {t2_space, topological_semigroup_mult, division_ring}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1448
  assumes \<open>c \<noteq> 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1449
  shows "(\<lambda>x. c * f x) summable_on A \<longleftrightarrow> f summable_on A"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  1450
    by (metis (no_types, lifting) assms left_inverse mult.assoc mult_1 summable_on_cmult_right summable_on_cong)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1451
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1452
lemma infsum_cmult_left':
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1453
  fixes f :: "'a \<Rightarrow> 'b :: {t2_space, topological_semigroup_mult, division_ring}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1454
  shows "infsum (\<lambda>x. f x * c) A = infsum f A * c"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1455
  by (metis (full_types) infsum_cmult_left infsum_not_exists mult_eq_0_iff summable_on_cmult_left')
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1456
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1457
lemma infsum_cmult_right':
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1458
  fixes f :: "'a \<Rightarrow> 'b :: {t2_space,topological_semigroup_mult,division_ring}"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1459
  shows "infsum (\<lambda>x. c * f x) A = c * infsum f A"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1460
  by (metis (full_types) infsum_cmult_right infsum_not_exists mult_eq_0_iff summable_on_cmult_right')
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1461
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1462
lemma has_sum_constant[simp]:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1463
  assumes \<open>finite F\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1464
  shows \<open>((\<lambda>_. c) has_sum of_nat (card F) * c) F\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1465
  by (metis assms has_sum_finite sum_constant)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1466
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1467
lemma infsum_constant[simp]:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1468
  assumes \<open>finite F\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1469
  shows \<open>infsum (\<lambda>_. c) F = of_nat (card F) * c\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1470
  by (simp add: assms)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1471
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1472
lemma infsum_diverge_constant:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1473
  \<comment> \<open>This probably does not really need all of \<^class>\<open>archimedean_field\<close> but Isabelle/HOL
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1474
       has no type class such as, e.g., "archimedean ring".\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1475
  fixes c :: \<open>'a::{archimedean_field, comm_monoid_add, linorder_topology, topological_semigroup_mult}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1476
  assumes \<open>infinite A\<close> and \<open>c \<noteq> 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1477
  shows \<open>\<not> (\<lambda>_. c) summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1478
proof (rule notI)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1479
  assume \<open>(\<lambda>_. c) summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1480
  then have \<open>(\<lambda>_. inverse c * c) summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1481
    by (rule summable_on_cmult_right)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1482
  then have [simp]: \<open>(\<lambda>_. 1::'a) summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1483
    using assms by auto
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1484
  have \<open>infsum (\<lambda>_. 1) A \<ge> d\<close> for d :: 'a
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1485
  proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1486
    obtain n :: nat where \<open>of_nat n \<ge> d\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1487
      by (meson real_arch_simple)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1488
    from assms
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1489
    obtain F where \<open>F \<subseteq> A\<close> and \<open>finite F\<close> and \<open>card F = n\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1490
      by (meson infinite_arbitrarily_large)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1491
    note \<open>d \<le> of_nat n\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1492
    also have \<open>of_nat n = infsum (\<lambda>_. 1::'a) F\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1493
      by (simp add: \<open>card F = n\<close> \<open>finite F\<close>)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1494
    also have \<open>\<dots> \<le> infsum (\<lambda>_. 1::'a) A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1495
      apply (rule infsum_mono_neutral)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1496
      using \<open>finite F\<close> \<open>F \<subseteq> A\<close> by auto
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1497
    finally show ?thesis .
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1498
  qed                                                        
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1499
  then show False
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1500
    by (meson linordered_field_no_ub not_less)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1501
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1502
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1503
lemma has_sum_constant_archimedean[simp]:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1504
  \<comment> \<open>This probably does not really need all of \<^class>\<open>archimedean_field\<close> but Isabelle/HOL
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1505
       has no type class such as, e.g., "archimedean ring".\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1506
  fixes c :: \<open>'a::{archimedean_field, comm_monoid_add, linorder_topology, topological_semigroup_mult}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1507
  shows \<open>infsum (\<lambda>_. c) A = of_nat (card A) * c\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1508
  by (metis infsum_0 infsum_constant infsum_diverge_constant infsum_not_exists sum.infinite sum_constant)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1509
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1510
lemma has_sum_uminus:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1511
  fixes f :: \<open>'a \<Rightarrow> 'b::topological_ab_group_add\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1512
  shows \<open>((\<lambda>x. - f x) has_sum a) A \<longleftrightarrow> (f has_sum (- a)) A\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1513
  by (auto simp add: sum_negf[abs_def] tendsto_minus_cancel_left has_sum_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1514
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1515
lemma summable_on_uminus:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1516
  fixes f :: \<open>'a \<Rightarrow> 'b::topological_ab_group_add\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1517
  shows\<open>(\<lambda>x. - f x) summable_on A \<longleftrightarrow> f summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1518
  by (metis summable_on_def has_sum_uminus verit_minus_simplify(4))
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1519
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1520
lemma infsum_uminus:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1521
  fixes f :: \<open>'a \<Rightarrow> 'b::{topological_ab_group_add, t2_space}\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1522
  shows \<open>infsum (\<lambda>x. - f x) A = - infsum f A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1523
  by (metis (full_types) add.inverse_inverse add.inverse_neutral infsumI infsum_def has_sum_infsum has_sum_uminus)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1524
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1525
lemma has_sum_le_finite_sums:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1526
  fixes a :: \<open>'a::{comm_monoid_add,topological_space,linorder_topology}\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1527
  assumes \<open>(f has_sum a) A\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1528
  assumes \<open>\<And>F. finite F \<Longrightarrow> F \<subseteq> A \<Longrightarrow> sum f F \<le> b\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1529
  shows \<open>a \<le> b\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1530
  by (metis assms eventually_finite_subsets_at_top_weakI finite_subsets_at_top_neq_bot has_sum_def tendsto_upperbound)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1531
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1532
lemma infsum_le_finite_sums:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1533
  fixes b :: \<open>'a::{comm_monoid_add,topological_space,linorder_topology}\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1534
  assumes \<open>f summable_on A\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1535
  assumes \<open>\<And>F. finite F \<Longrightarrow> F \<subseteq> A \<Longrightarrow> sum f F \<le> b\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1536
  shows \<open>infsum f A \<le> b\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1537
  by (meson assms has_sum_infsum has_sum_le_finite_sums)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1538
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1539
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1540
lemma summable_on_scaleR_left [intro]:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1541
  fixes c :: \<open>'a :: real_normed_vector\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1542
  assumes "c \<noteq> 0 \<Longrightarrow> f summable_on A"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1543
  shows   "(\<lambda>x. f x *\<^sub>R c) summable_on A"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1544
proof (cases \<open>c = 0\<close>)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1545
  case False
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1546
  then have "(\<lambda>y. y *\<^sub>R c) \<circ> f summable_on A"
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1547
    using assms by (auto simp add: scaleR_left.additive_axioms summable_on_comm_additive)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1548
  then show ?thesis
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1549
    by (metis (mono_tags, lifting) comp_apply summable_on_cong)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1550
qed auto
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1551
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1552
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1553
lemma summable_on_scaleR_right [intro]:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1554
  fixes f :: \<open>'a \<Rightarrow> 'b :: real_normed_vector\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1555
  assumes "c \<noteq> 0 \<Longrightarrow> f summable_on A"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1556
  shows   "(\<lambda>x. c *\<^sub>R f x) summable_on A"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1557
proof (cases \<open>c = 0\<close>)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1558
  case False
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1559
  then have "(*\<^sub>R) c \<circ> f summable_on A"
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1560
  using assms by (auto simp add: scaleR_right.additive_axioms summable_on_comm_additive)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1561
  then show ?thesis
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1562
    by (metis (mono_tags, lifting) comp_apply summable_on_cong)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1563
qed auto
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1564
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1565
lemma infsum_scaleR_left:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1566
  fixes c :: \<open>'a :: real_normed_vector\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1567
  assumes "c \<noteq> 0 \<Longrightarrow> f summable_on A"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1568
  shows   "infsum (\<lambda>x. f x *\<^sub>R c) A = infsum f A *\<^sub>R c"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1569
proof (cases \<open>c = 0\<close>)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1570
  case False
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1571
  then have "infsum ((\<lambda>y. y *\<^sub>R c) \<circ> f) A = infsum f A *\<^sub>R c"
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1572
  using assms by (auto simp add: scaleR_left.additive_axioms infsum_comm_additive)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1573
  then show ?thesis
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1574
    by (metis (mono_tags, lifting) comp_apply infsum_cong)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1575
qed auto
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1576
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1577
lemma infsum_scaleR_right:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1578
  fixes f :: \<open>'a \<Rightarrow> 'b :: real_normed_vector\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1579
  shows   "infsum (\<lambda>x. c *\<^sub>R f x) A = c *\<^sub>R infsum f A"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1580
proof -
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1581
  consider (summable) \<open>f summable_on A\<close> | (c0) \<open>c = 0\<close> | (not_summable) \<open>\<not> f summable_on A\<close> \<open>c \<noteq> 0\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1582
    by auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1583
  then show ?thesis
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1584
  proof cases
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1585
    case summable
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1586
    then have "infsum ((*\<^sub>R) c \<circ> f) A = c *\<^sub>R infsum f A"
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1587
      by (auto simp add: scaleR_right.additive_axioms infsum_comm_additive)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1588
    then show ?thesis
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1589
      by (metis (mono_tags, lifting) comp_apply infsum_cong)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1590
  next
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1591
    case c0
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1592
    then show ?thesis by auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1593
  next
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1594
    case not_summable
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1595
    have \<open>\<not> (\<lambda>x. c *\<^sub>R f x) summable_on A\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1596
    proof (rule notI)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1597
      assume \<open>(\<lambda>x. c *\<^sub>R f x) summable_on A\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1598
      then have \<open>(\<lambda>x. inverse c *\<^sub>R c *\<^sub>R f x) summable_on A\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1599
        using summable_on_scaleR_right by blast
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1600
      with not_summable show False
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1601
        by simp
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1602
    qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1603
    then show ?thesis
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1604
      by (simp add: infsum_not_exists not_summable(1)) 
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1605
  qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1606
qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1607
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1608
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1609
lemma infsum_Un_Int:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1610
  fixes f :: "'a \<Rightarrow> 'b::{topological_ab_group_add, t2_space}"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1611
  assumes "f summable_on A - B" "f summable_on B - A" \<open>f summable_on A \<inter> B\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1612
  shows   "infsum f (A \<union> B) = infsum f A + infsum f B - infsum f (A \<inter> B)"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1613
proof -
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1614
  obtain \<open>f summable_on A\<close> \<open>f summable_on B\<close>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1615
    using assms by (metis Int_Diff_Un Int_Diff_disjoint inf_commute summable_on_Un_disjoint)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1616
  then have \<open>infsum f (A \<union> B) = infsum f A + infsum f (B - A)\<close>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1617
    using assms(2) infsum_Un_disjoint by fastforce
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1618
  moreover have \<open>infsum f (B - A) = infsum f B - infsum f (A \<inter> B)\<close>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1619
    using assms by (metis Diff_Int2 Un_Int_eq(2) \<open>f summable_on B\<close> inf_le2 infsum_Diff)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1620
  ultimately show ?thesis
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1621
    by auto
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1622
qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1623
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1624
lemma inj_combinator':
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1625
  assumes "x \<notin> F"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1626
  shows \<open>inj_on (\<lambda>(g, y). g(x := y)) (Pi\<^sub>E F B \<times> B x)\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1627
proof -
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1628
  have "inj_on ((\<lambda>(y, g). g(x := y)) \<circ> prod.swap) (Pi\<^sub>E F B \<times> B x)"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1629
    using inj_combinator[of x F B] assms by (intro comp_inj_on) (auto simp: product_swap)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1630
  thus ?thesis
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1631
    by (simp add: o_def)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1632
qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1633
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1634
lemma infsum_prod_PiE:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1635
  \<comment> \<open>See also \<open>infsum_prod_PiE_abs\<close> below with incomparable premises.\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1636
  fixes f :: "'a \<Rightarrow> 'b \<Rightarrow> 'c :: {comm_monoid_mult, topological_semigroup_mult, division_ring, banach}"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1637
  assumes finite: "finite A"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1638
  assumes "\<And>x. x \<in> A \<Longrightarrow> f x summable_on B x"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1639
  assumes "(\<lambda>g. \<Prod>x\<in>A. f x (g x)) summable_on (PiE A B)"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1640
  shows   "infsum (\<lambda>g. \<Prod>x\<in>A. f x (g x)) (PiE A B) = (\<Prod>x\<in>A. infsum (f x) (B x))"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1641
proof (use finite assms(2-) in induction)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1642
  case empty
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1643
  then show ?case 
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1644
    by auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1645
next
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1646
  case (insert x F)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1647
  have pi: \<open>Pi\<^sub>E (insert x F) B = (\<lambda>(g,y). g(x:=y)) ` (Pi\<^sub>E F B \<times> B x)\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1648
    unfolding PiE_insert_eq 
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1649
    by (subst swap_product [symmetric]) (simp add: image_image case_prod_unfold)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1650
  have prod: \<open>(\<Prod>x'\<in>F. f x' ((p(x:=y)) x')) = (\<Prod>x'\<in>F. f x' (p x'))\<close> for p y
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1651
    by (rule prod.cong) (use insert.hyps in auto)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1652
  have inj: \<open>inj_on (\<lambda>(g, y). g(x := y)) (Pi\<^sub>E F B \<times> B x)\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1653
    using \<open>x \<notin> F\<close> by (rule inj_combinator')
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1654
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1655
  have summable1: \<open>(\<lambda>g. \<Prod>x\<in>insert x F. f x (g x)) summable_on Pi\<^sub>E (insert x F) B\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1656
    using insert.prems(2) .
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1657
  also have \<open>Pi\<^sub>E (insert x F) B = (\<lambda>(g,y). g(x:=y)) ` (Pi\<^sub>E F B \<times> B x)\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1658
    by (simp only: pi)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1659
  also have "(\<lambda>g. \<Prod>x\<in>insert x F. f x (g x)) summable_on \<dots> \<longleftrightarrow>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1660
               ((\<lambda>g. \<Prod>x\<in>insert x F. f x (g x)) \<circ> (\<lambda>(g,y). g(x:=y))) summable_on (Pi\<^sub>E F B \<times> B x)"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1661
    using inj by (rule summable_on_reindex)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1662
  also have "(\<Prod>z\<in>F. f z ((g(x := y)) z)) = (\<Prod>z\<in>F. f z (g z))" for g y
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1663
    using insert.hyps by (intro prod.cong) auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1664
  hence "((\<lambda>g. \<Prod>x\<in>insert x F. f x (g x)) \<circ> (\<lambda>(g,y). g(x:=y))) =
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1665
             (\<lambda>(p, y). f x y * (\<Prod>x'\<in>F. f x' (p x')))"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1666
    using insert.hyps by (auto simp: fun_eq_iff cong: prod.cong_simp)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1667
  finally have summable2: \<open>(\<lambda>(p, y). f x y * (\<Prod>x'\<in>F. f x' (p x'))) summable_on Pi\<^sub>E F B \<times> B x\<close> .
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1668
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1669
  then have \<open>(\<lambda>p. \<Sum>\<^sub>\<infinity>y\<in>B x. f x y * (\<Prod>x'\<in>F. f x' (p x'))) summable_on Pi\<^sub>E F B\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1670
    by (rule summable_on_Sigma_banach)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1671
  then have \<open>(\<lambda>p. (\<Sum>\<^sub>\<infinity>y\<in>B x. f x y) * (\<Prod>x'\<in>F. f x' (p x'))) summable_on Pi\<^sub>E F B\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1672
    by (metis (mono_tags, lifting) infsum_cmult_left' infsum_cong summable_on_cong)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1673
  then have summable3: \<open>(\<lambda>p. (\<Prod>x'\<in>F. f x' (p x'))) summable_on Pi\<^sub>E F B\<close> if \<open>(\<Sum>\<^sub>\<infinity>y\<in>B x. f x y) \<noteq> 0\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1674
    using summable_on_cmult_right' that by blast
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1675
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1676
  have \<open>(\<Sum>\<^sub>\<infinity>g\<in>Pi\<^sub>E (insert x F) B. \<Prod>x\<in>insert x F. f x (g x))
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1677
     = (\<Sum>\<^sub>\<infinity>(p,y)\<in>Pi\<^sub>E F B \<times> B x. \<Prod>x'\<in>insert x F. f x' ((p(x:=y)) x'))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1678
    by (smt (verit, ccfv_SIG) comp_apply infsum_cong infsum_reindex inj pi prod.cong split_def)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1679
  also have \<open>\<dots> = (\<Sum>\<^sub>\<infinity>(p, y)\<in>Pi\<^sub>E F B \<times> B x. f x y * (\<Prod>x'\<in>F. f x' ((p(x:=y)) x')))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1680
    using insert.hyps by auto
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1681
  also have \<open>\<dots> = (\<Sum>\<^sub>\<infinity>(p, y)\<in>Pi\<^sub>E F B \<times> B x. f x y * (\<Prod>x'\<in>F. f x' (p x')))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1682
    using prod by presburger
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1683
  also have \<open>\<dots> = (\<Sum>\<^sub>\<infinity>p\<in>Pi\<^sub>E F B. \<Sum>\<^sub>\<infinity>y\<in>B x. f x y * (\<Prod>x'\<in>F. f x' (p x')))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1684
    using infsum_Sigma'_banach summable2 by force
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1685
  also have \<open>\<dots> = (\<Sum>\<^sub>\<infinity>y\<in>B x. f x y) * (\<Sum>\<^sub>\<infinity>p\<in>Pi\<^sub>E F B. \<Prod>x'\<in>F. f x' (p x'))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1686
    by (smt (verit) infsum_cmult_left' infsum_cmult_right' infsum_cong)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1687
  also have \<open>\<dots> = (\<Prod>x\<in>insert x F. infsum (f x) (B x))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1688
    using insert summable3 by auto
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1689
  finally show ?case
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1690
    by simp
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1691
qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1692
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1693
lemma infsum_prod_PiE_abs:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1694
  \<comment> \<open>See also @{thm [source] infsum_prod_PiE} above with incomparable premises.\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1695
  fixes f :: "'a \<Rightarrow> 'b \<Rightarrow> 'c :: {banach, real_normed_div_algebra, comm_semiring_1}"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1696
  assumes finite: "finite A"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1697
  assumes "\<And>x. x \<in> A \<Longrightarrow> f x abs_summable_on B x"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1698
  shows   "infsum (\<lambda>g. \<Prod>x\<in>A. f x (g x)) (PiE A B) = (\<Prod>x\<in>A. infsum (f x) (B x))"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1699
proof (use finite assms(2) in induction)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1700
  case empty
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1701
  then show ?case 
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1702
    by auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1703
next
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1704
  case (insert x A)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1705
  
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1706
  have pi: \<open>Pi\<^sub>E (insert x F) B = (\<lambda>(g,y). g(x:=y)) ` (Pi\<^sub>E F B \<times> B x)\<close> for x F and B :: "'a \<Rightarrow> 'b set"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1707
    unfolding PiE_insert_eq 
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1708
    by (subst swap_product [symmetric]) (simp add: image_image case_prod_unfold)
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1709
  have prod: \<open>(\<Prod>x'\<in>A. f x' ((p(x:=y)) x')) = (\<Prod>x'\<in>A. f x' (p x'))\<close> for p y
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1710
    by (rule prod.cong) (use insert.hyps in auto)
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1711
  have inj: \<open>inj_on (\<lambda>(g, y). g(x := y)) (Pi\<^sub>E A B \<times> B x)\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1712
    using \<open>x \<notin> A\<close> by (rule inj_combinator')
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1713
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1714
  define s where \<open>s x = infsum (\<lambda>y. norm (f x y)) (B x)\<close> for x
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1715
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1716
  have \<open>(\<Sum>p\<in>P. norm (\<Prod>x\<in>F. f x (p x))) \<le> prod s F\<close> 
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1717
    if P: \<open>P \<subseteq> Pi\<^sub>E F B\<close> and [simp]: \<open>finite P\<close> \<open>finite F\<close> 
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1718
      and sum: \<open>\<And>x. x \<in> F \<Longrightarrow> f x abs_summable_on B x\<close> for P F
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1719
  proof -
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1720
    define B' where \<open>B' x = {p x| p. p\<in>P}\<close> for x
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1721
    have fin_B'[simp]: \<open>finite (B' x)\<close> for x
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1722
      using that by (auto simp: B'_def)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1723
    have [simp]: \<open>finite (Pi\<^sub>E F B')\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1724
      by (simp add: finite_PiE)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1725
    have [simp]: \<open>P \<subseteq> Pi\<^sub>E F B'\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1726
      using that by (auto simp: B'_def)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1727
    have B'B: \<open>B' x \<subseteq> B x\<close> if \<open>x \<in> F\<close> for x
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1728
      unfolding B'_def using P that 
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1729
      by auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1730
    have s_bound: \<open>(\<Sum>y\<in>B' x. norm (f x y)) \<le> s x\<close> if \<open>x \<in> F\<close> for x
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1731
      by (metis B'B fin_B' finite_sum_le_has_sum has_sum_infsum norm_ge_zero s_def sum that)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1732
    have \<open>(\<Sum>p\<in>P. norm (\<Prod>x\<in>F. f x (p x))) \<le> (\<Sum>p\<in>Pi\<^sub>E F B'. norm (\<Prod>x\<in>F. f x (p x)))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1733
      by (simp add: sum_mono2)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1734
    also have \<open>\<dots> = (\<Sum>p\<in>Pi\<^sub>E F B'. \<Prod>x\<in>F. norm (f x (p x)))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1735
      by (simp add: prod_norm)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1736
    also have \<open>\<dots> = (\<Prod>x\<in>F. \<Sum>y\<in>B' x. norm (f x y))\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1737
    proof (use \<open>finite F\<close> in induction)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1738
      case empty
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1739
      then show ?case by simp
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1740
    next
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1741
      case (insert x F)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1742
      have inj: \<open>inj_on (\<lambda>(g, y). g(x := y)) (Pi\<^sub>E F B' \<times> B' x)\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1743
        by (simp add: inj_combinator' insert.hyps)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1744
      then have \<open>(\<Sum>p\<in>Pi\<^sub>E (insert x F) B'. \<Prod>x\<in>insert x F. norm (f x (p x)))
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1745
         =  (\<Sum>(p,y)\<in>Pi\<^sub>E F B' \<times> B' x. \<Prod>x'\<in>insert x F. norm (f x' ((p(x := y)) x')))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1746
        by (simp add: pi sum.reindex case_prod_unfold)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1747
      also have \<open>\<dots> = (\<Sum>(p, y)\<in>Pi\<^sub>E F B' \<times> B' x. norm (f x y) * (\<Prod>x'\<in>F. norm (f x' (p x'))))\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1748
        by (smt (verit, del_insts) fun_upd_apply insert.hyps prod.cong prod.insert split_def sum.cong)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1749
      also have \<open>\<dots> = (\<Sum>y\<in>B' x. norm (f x y)) * (\<Sum>p\<in>Pi\<^sub>E F B'. \<Prod>x'\<in>F. norm (f x' (p x')))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1750
        by (simp add: sum_product sum.swap [of _ "Pi\<^sub>E F B'"] sum.cartesian_product)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1751
      also have \<open>\<dots> = (\<Prod>x\<in>insert x F. \<Sum>y\<in>B' x. norm (f x y))\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1752
        using insert by force
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1753
      finally show ?case .
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1754
    qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1755
    also have \<open>\<dots> \<le> (\<Prod>x\<in>F. s x)\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1756
      using s_bound by (simp add: prod_mono sum_nonneg)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1757
    finally show ?thesis .
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1758
  qed
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1759
  then have "bdd_above
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1760
     (sum (\<lambda>g. norm (\<Prod>x\<in>insert x A. f x (g x))) ` {F. F \<subseteq> Pi\<^sub>E (insert x A) B \<and> finite F})"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1761
    using insert.hyps insert.prems by (intro bdd_aboveI) blast
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1762
  then have \<open>(\<lambda>g. \<Prod>x\<in>insert x A. f x (g x)) abs_summable_on Pi\<^sub>E (insert x A) B\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1763
    using nonneg_bdd_above_summable_on
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1764
    by (metis (mono_tags, lifting) Collect_cong norm_ge_zero)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1765
  also have \<open>Pi\<^sub>E (insert x A) B = (\<lambda>(g,y). g(x:=y)) ` (Pi\<^sub>E A B \<times> B x)\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1766
    by (simp only: pi)
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1767
  also have "(\<lambda>g. \<Prod>x\<in>insert x A. f x (g x)) abs_summable_on \<dots> \<longleftrightarrow>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1768
               ((\<lambda>g. \<Prod>x\<in>insert x A. f x (g x)) \<circ> (\<lambda>(g,y). g(x:=y))) abs_summable_on (Pi\<^sub>E A B \<times> B x)"
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1769
    using inj by (subst summable_on_reindex) (auto simp: o_def)
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1770
  also have "(\<Prod>z\<in>A. f z ((g(x := y)) z)) = (\<Prod>z\<in>A. f z (g z))" for g y
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1771
    using insert.hyps by (intro prod.cong) auto
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1772
  hence "((\<lambda>g. \<Prod>x\<in>insert x A. f x (g x)) \<circ> (\<lambda>(g,y). g(x:=y))) =
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1773
             (\<lambda>(p, y). f x y * (\<Prod>x'\<in>A. f x' (p x')))"
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1774
    using insert.hyps by (auto simp: fun_eq_iff cong: prod.cong_simp)
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1775
  finally have summable2: \<open>(\<lambda>(p, y). f x y * (\<Prod>x'\<in>A. f x' (p x'))) abs_summable_on Pi\<^sub>E A B \<times> B x\<close> .
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1776
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1777
  have \<open>(\<Sum>\<^sub>\<infinity>g\<in>Pi\<^sub>E (insert x A) B. \<Prod>x\<in>insert x A. f x (g x))
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1778
     = (\<Sum>\<^sub>\<infinity>(p,y)\<in>Pi\<^sub>E A B \<times> B x. \<Prod>x'\<in>insert x A. f x' ((p(x:=y)) x'))\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1779
    using inj by (simp add: pi infsum_reindex o_def case_prod_unfold)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1780
  also have \<open>\<dots> = (\<Sum>\<^sub>\<infinity>(p,y) \<in> Pi\<^sub>E A B \<times> B x. f x y * (\<Prod>x'\<in>A. f x' (p x')))\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1781
    using prod insert.hyps by auto
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1782
  also have \<open>\<dots> = (\<Sum>\<^sub>\<infinity>p\<in>Pi\<^sub>E A B. \<Sum>\<^sub>\<infinity>y\<in>B x. f x y * (\<Prod>x'\<in>A. f x' (p x')))\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1783
    using abs_summable_summable infsum_Sigma'_banach summable2 by fastforce
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1784
  also have \<open>\<dots> = (\<Sum>\<^sub>\<infinity>y\<in>B x. f x y) * (\<Sum>\<^sub>\<infinity>p\<in>Pi\<^sub>E A B. \<Prod>x'\<in>A. f x' (p x'))\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1785
    by (smt (verit, best) infsum_cmult_left' infsum_cmult_right' infsum_cong)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1786
  finally show ?case
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1787
    by (simp add: insert)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1788
qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1789
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1790
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1792
subsection \<open>Absolute convergence\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1793
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1794
lemma abs_summable_countable:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1795
  assumes \<open>f abs_summable_on A\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1796
  shows \<open>countable {x\<in>A. f x \<noteq> 0}\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1797
proof -
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1798
  have fin: \<open>finite {x\<in>A. norm (f x) \<ge> t}\<close> if \<open>t > 0\<close> for t
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1799
  proof (rule ccontr)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1800
    assume *: \<open>infinite {x \<in> A. t \<le> norm (f x)}\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1801
    have \<open>infsum (\<lambda>x. norm (f x)) A \<ge> b\<close> for b
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1802
    proof -
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1803
      obtain b' where b': \<open>of_nat b' \<ge> b / t\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1804
        by (meson real_arch_simple)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1805
      from *
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1806
      obtain F where cardF: \<open>card F \<ge> b'\<close> and \<open>finite F\<close> and F: \<open>F \<subseteq> {x \<in> A. t \<le> norm (f x)}\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1807
        by (meson finite_if_finite_subsets_card_bdd nle_le)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1808
      have \<open>b \<le> of_nat b' * t\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1809
        using b' \<open>t > 0\<close> by (simp add: field_simps split: if_splits)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1810
      also have \<open>\<dots> \<le> of_nat (card F) * t\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1811
        by (simp add: cardF that)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1812
      also have \<open>\<dots> = sum (\<lambda>x. t) F\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1813
        by simp
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1814
      also have \<open>\<dots> \<le> sum (\<lambda>x. norm (f x)) F\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1815
        by (metis (mono_tags, lifting) F in_mono mem_Collect_eq sum_mono)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1816
      also have \<open>\<dots> = infsum (\<lambda>x. norm (f x)) F\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1817
        using \<open>finite F\<close> by (rule infsum_finite[symmetric])
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1818
      also have \<open>\<dots> \<le> infsum (\<lambda>x. norm (f x)) A\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1819
        by (rule infsum_mono_neutral) (use \<open>finite F\<close> assms F in auto)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1820
      finally show ?thesis .
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1821
    qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1822
    then show False
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1823
      by (meson gt_ex linorder_not_less)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1824
  qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1825
  have \<open>countable (\<Union>i\<in>{1..}. {x\<in>A. norm (f x) \<ge> 1/of_nat i})\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1826
    by (rule countable_UN) (use fin in \<open>auto intro!: countable_finite\<close>)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1827
  also have \<open>\<dots> = {x\<in>A. f x \<noteq> 0}\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1828
  proof safe
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1829
    fix x assume x: "x \<in> A" "f x \<noteq> 0"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1830
    define i where "i = max 1 (nat (ceiling (1 / norm (f x))))"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1831
    have "i \<ge> 1"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1832
      by (simp add: i_def)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1833
    moreover have "real i \<ge> 1 / norm (f x)"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1834
      unfolding i_def by linarith
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1835
    hence "1 / real i \<le> norm (f x)" using \<open>f x \<noteq> 0\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1836
      by (auto simp: divide_simps mult_ac)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1837
    ultimately show "x \<in> (\<Union>i\<in>{1..}. {x \<in> A. 1 / real i \<le> norm (f x)})"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1838
      using \<open>x \<in> A\<close> by auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1839
  qed auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1840
  finally show ?thesis .
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1841
qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1842
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1843
(* Logically belongs in the section about reals, but needed as a dependency here *)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1844
lemma summable_on_iff_abs_summable_on_real:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1845
  fixes f :: \<open>'a \<Rightarrow> real\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1846
  shows \<open>f summable_on A \<longleftrightarrow> f abs_summable_on A\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1847
proof (rule iffI)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1848
  assume \<open>f summable_on A\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1849
  define n A\<^sub>p A\<^sub>n
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1850
    where \<open>n \<equiv> \<lambda>x. norm (f x)\<close> and \<open>A\<^sub>p = {x\<in>A. f x \<ge> 0}\<close> and \<open>A\<^sub>n = {x\<in>A. f x < 0}\<close> for x
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1851
  have A: \<open>A\<^sub>p \<union> A\<^sub>n = A\<close> \<open>A\<^sub>p \<inter> A\<^sub>n = {}\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1852
    by (auto simp: A\<^sub>p_def A\<^sub>n_def)
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1853
  from \<open>f summable_on A\<close> have \<open>f summable_on A\<^sub>p\<close> \<open>f summable_on A\<^sub>n\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1854
    using A\<^sub>p_def A\<^sub>n_def summable_on_subset_banach by fastforce+
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1855
  then have \<open>n summable_on A\<^sub>p\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1856
    by (smt (verit) A\<^sub>p_def n_def mem_Collect_eq real_norm_def summable_on_cong)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1857
  moreover have \<open>n summable_on A\<^sub>n\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1858
    by (smt (verit, best) \<open>f summable_on A\<^sub>n\<close>  summable_on_uminus A\<^sub>n_def n_def summable_on_cong mem_Collect_eq real_norm_def)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1859
  ultimately show \<open>n summable_on A\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1860
    using A summable_on_Un_disjoint by blast
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1861
next
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1862
  show \<open>f abs_summable_on A \<Longrightarrow> f summable_on A\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1863
    using abs_summable_summable by blast
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1864
qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1865
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1866
lemma abs_summable_on_Sigma_iff:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1867
  shows   "f abs_summable_on Sigma A B \<longleftrightarrow>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1868
             (\<forall>x\<in>A. (\<lambda>y. f (x, y)) abs_summable_on B x) \<and>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1869
             ((\<lambda>x. infsum (\<lambda>y. norm (f (x, y))) (B x)) abs_summable_on A)"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1870
proof (intro iffI conjI ballI)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1871
  assume asm: \<open>f abs_summable_on Sigma A B\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1872
  then have \<open>(\<lambda>x. infsum (\<lambda>y. norm (f (x,y))) (B x)) summable_on A\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1873
    by (simp add: cond_case_prod_eta summable_on_Sigma_banach)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1874
  then show \<open>(\<lambda>x. \<Sum>\<^sub>\<infinity>y\<in>B x. norm (f (x, y))) abs_summable_on A\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1875
    using summable_on_iff_abs_summable_on_real by force
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1876
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1877
  show \<open>(\<lambda>y. f (x, y)) abs_summable_on B x\<close> if \<open>x \<in> A\<close> for x
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1878
  proof -
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1879
    from asm have \<open>f abs_summable_on Pair x ` B x\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1880
      by (simp add: image_subset_iff summable_on_subset_banach that)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1881
    then show ?thesis
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1882
      by (metis (mono_tags, lifting) o_def inj_on_def summable_on_reindex prod.inject summable_on_cong)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1883
  qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1884
next
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1885
  assume asm: \<open>(\<forall>x\<in>A. (\<lambda>xa. f (x, xa)) abs_summable_on B x) \<and>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1886
    (\<lambda>x. \<Sum>\<^sub>\<infinity>y\<in>B x. norm (f (x, y))) abs_summable_on A\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1887
  have \<open>(\<Sum>xy\<in>F. norm (f xy)) \<le> (\<Sum>\<^sub>\<infinity>x\<in>A. \<Sum>\<^sub>\<infinity>y\<in>B x. norm (f (x, y)))\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1888
    if \<open>F \<subseteq> Sigma A B\<close> and [simp]: \<open>finite F\<close> for F
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1889
  proof -
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1890
    have [simp]: \<open>(SIGMA x:fst ` F. {y. (x, y) \<in> F}) = F\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1891
      by (auto intro!: set_eqI simp add: Domain.DomainI fst_eq_Domain)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1892
    have [simp]: \<open>finite {y. (x, y) \<in> F}\<close> for x
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1893
      by (metis \<open>finite F\<close> Range.intros finite_Range finite_subset mem_Collect_eq subsetI)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1894
    have \<open>(\<Sum>xy\<in>F. norm (f xy)) = (\<Sum>x\<in>fst ` F. \<Sum>y\<in>{y. (x,y)\<in>F}. norm (f (x,y)))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1895
      by (simp add: sum.Sigma)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1896
    also have \<open>\<dots> = (\<Sum>\<^sub>\<infinity>x\<in>fst ` F. \<Sum>\<^sub>\<infinity>y\<in>{y. (x,y)\<in>F}. norm (f (x,y)))\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1897
      by auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1898
    also have \<open>\<dots> \<le> (\<Sum>\<^sub>\<infinity>x\<in>fst ` F. \<Sum>\<^sub>\<infinity>y\<in>B x. norm (f (x,y)))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1899
      using asm that(1) by (intro infsum_mono infsum_mono_neutral) auto
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1900
    also have \<open>\<dots> \<le> (\<Sum>\<^sub>\<infinity>x\<in>A. \<Sum>\<^sub>\<infinity>y\<in>B x. norm (f (x,y)))\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1901
      by (rule infsum_mono_neutral) (use asm that(1) in \<open>auto simp add: infsum_nonneg\<close>)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1902
    finally show ?thesis .
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1903
  qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1904
  then show \<open>f abs_summable_on Sigma A B\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1905
    by (intro nonneg_bdd_above_summable_on) (auto simp: bdd_above_def)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1906
qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1907
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1908
lemma abs_summable_on_comparison_test:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1909
  assumes "g abs_summable_on A"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1910
  assumes "\<And>x. x \<in> A \<Longrightarrow> norm (f x) \<le> norm (g x)"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1911
  shows   "f abs_summable_on A"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1912
proof (rule nonneg_bdd_above_summable_on)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1913
  show "bdd_above (sum (\<lambda>x. norm (f x)) ` {F. F \<subseteq> A \<and> finite F})"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1914
  proof (rule bdd_aboveI2)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1915
    fix F assume F: "F \<in> {F. F \<subseteq> A \<and> finite F}"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1916
    have \<open>sum (\<lambda>x. norm (f x)) F \<le> sum (\<lambda>x. norm (g x)) F\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1917
      using assms F by (intro sum_mono) auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1918
    also have \<open>\<dots> = infsum (\<lambda>x. norm (g x)) F\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1919
      using F by simp
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1920
    also have \<open>\<dots> \<le> infsum (\<lambda>x. norm (g x)) A\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1921
      by (smt (verit) F assms(1) infsum_mono2 mem_Collect_eq norm_ge_zero summable_on_subset_banach)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1922
    finally show "(\<Sum>x\<in>F. norm (f x)) \<le> (\<Sum>\<^sub>\<infinity>x\<in>A. norm (g x))" .
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1923
  qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1924
qed auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1925
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1926
lemma abs_summable_iff_bdd_above:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1927
  fixes f :: \<open>'a \<Rightarrow> 'b::real_normed_vector\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1928
  shows \<open>f abs_summable_on A \<longleftrightarrow> bdd_above (sum (\<lambda>x. norm (f x)) ` {F. F\<subseteq>A \<and> finite F})\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1929
proof (rule iffI)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1930
  assume \<open>f abs_summable_on A\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1931
  show \<open>bdd_above (sum (\<lambda>x. norm (f x)) ` {F. F \<subseteq> A \<and> finite F})\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1932
  proof (rule bdd_aboveI2)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1933
    fix F assume F: "F \<in> {F. F \<subseteq> A \<and> finite F}"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1934
    show "(\<Sum>x\<in>F. norm (f x)) \<le> (\<Sum>\<^sub>\<infinity>x\<in>A. norm (f x))"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1935
      by (rule finite_sum_le_infsum) (use \<open>f abs_summable_on A\<close> F in auto)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1936
  qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1937
next
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1938
  assume \<open>bdd_above (sum (\<lambda>x. norm (f x)) ` {F. F\<subseteq>A \<and> finite F})\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1939
  then show \<open>f abs_summable_on A\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1940
    by (simp add: nonneg_bdd_above_summable_on)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1941
qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1942
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1943
lemma abs_summable_product:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1944
  fixes x :: "'a \<Rightarrow> 'b::{real_normed_div_algebra,banach,second_countable_topology}"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1945
  assumes x2_sum: "(\<lambda>i. (x i) * (x i)) abs_summable_on A"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1946
    and y2_sum: "(\<lambda>i. (y i) * (y i)) abs_summable_on A"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1947
  shows "(\<lambda>i. x i * y i) abs_summable_on A"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1948
proof (rule nonneg_bdd_above_summable_on)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1949
  show "bdd_above (sum (\<lambda>xa. norm (x xa * y xa)) ` {F. F \<subseteq> A \<and> finite F})"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1950
  proof (rule bdd_aboveI2)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1951
    fix F assume F: \<open>F \<in> {F. F \<subseteq> A \<and> finite F}\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1952
    then have r1: "finite F" and b4: "F \<subseteq> A"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1953
      by auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1954
  
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1955
    have a1: "(\<Sum>\<^sub>\<infinity>i\<in>F. norm (x i * x i)) \<le> (\<Sum>\<^sub>\<infinity>i\<in>A. norm (x i * x i))"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1956
      by (metis (no_types, lifting) b4 infsum_mono2 norm_ge_zero summable_on_subset_banach x2_sum)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1957
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1958
    have "norm (x i * y i) \<le> norm (x i * x i) + norm (y i * y i)" for i
79757
f20ac6788faa tuned proof: avoid z3 to make it work on arm64-linux;
wenzelm
parents: 79529
diff changeset
  1959
      unfolding norm_mult by (smt (verit, best) abs_norm_cancel mult_mono not_sum_squares_lt_zero)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1960
    hence "(\<Sum>i\<in>F. norm (x i * y i)) \<le> (\<Sum>i\<in>F. norm (x i * x i) + norm (y i * y i))"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1961
      by (simp add: sum_mono)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1962
    also have "\<dots> = (\<Sum>i\<in>F. norm (x i * x i)) + (\<Sum>i\<in>F. norm (y i * y i))"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1963
      by (simp add: sum.distrib)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1964
    also have "\<dots> = (\<Sum>\<^sub>\<infinity>i\<in>F. norm (x i * x i)) + (\<Sum>\<^sub>\<infinity>i\<in>F. norm (y i * y i))"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1965
      by (simp add: \<open>finite F\<close>)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1966
    also have "\<dots> \<le> (\<Sum>\<^sub>\<infinity>i\<in>A. norm (x i * x i)) + (\<Sum>\<^sub>\<infinity>i\<in>A. norm (y i * y i))"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1967
      using F assms
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1968
      by (intro add_mono infsum_mono2) auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1969
    finally show \<open>(\<Sum>xa\<in>F. norm (x xa * y xa)) \<le> (\<Sum>\<^sub>\<infinity>i\<in>A. norm (x i * x i)) + (\<Sum>\<^sub>\<infinity>i\<in>A. norm (y i * y i))\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1970
      by simp
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1971
  qed
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1972
qed auto
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  1973
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1974
subsection \<open>Extended reals and nats\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1975
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1976
lemma summable_on_ennreal[simp]: \<open>(f::_ \<Rightarrow> ennreal) summable_on S\<close> and summable_on_enat[simp]: \<open>(f::_ \<Rightarrow> enat) summable_on S\<close>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1977
  by (simp_all add: nonneg_summable_on_complete)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1978
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1979
lemma has_sum_superconst_infinite_ennreal:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1980
  fixes f :: \<open>'a \<Rightarrow> ennreal\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1981
  assumes geqb: \<open>\<And>x. x \<in> S \<Longrightarrow> f x \<ge> b\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1982
  assumes b: \<open>b > 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1983
  assumes \<open>infinite S\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  1984
  shows "(f has_sum \<infinity>) S"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1985
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1986
  have \<open>(sum f \<longlongrightarrow> \<infinity>) (finite_subsets_at_top S)\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1987
  proof (rule order_tendstoI)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1988
    fix y :: ennreal assume \<open>y < \<infinity>\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1989
    then have \<open>y / b < \<infinity>\<close> \<open>y < top\<close>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1990
      using b ennreal_divide_eq_top_iff top.not_eq_extremum by force+
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1991
    then obtain F where \<open>finite F\<close> and \<open>F \<subseteq> S\<close> and cardF: \<open>card F > y / b\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1992
      using \<open>infinite S\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1993
      by (metis ennreal_Ex_less_of_nat infinite_arbitrarily_large infinity_ennreal_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1994
    moreover have \<open>sum f Y > y\<close> if \<open>finite Y\<close> and \<open>F \<subseteq> Y\<close> and \<open>Y \<subseteq> S\<close> for Y
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1995
    proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1996
      have \<open>y < b * card F\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1997
        by (metis b \<open>y < top\<close> cardF divide_less_ennreal ennreal_mult_eq_top_iff gr_implies_not_zero mult.commute top.not_eq_extremum)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  1998
      also have \<open>\<dots> \<le> b * card Y\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  1999
        by (meson b card_mono less_imp_le mult_left_mono of_nat_le_iff that)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2000
      also have \<open>\<dots> = sum (\<lambda>_. b) Y\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2001
        by (simp add: mult.commute)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2002
      also have \<open>\<dots> \<le> sum f Y\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2003
        using geqb by (meson subset_eq sum_mono that(3))
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2004
      finally show ?thesis .
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2005
    qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2006
    ultimately show \<open>\<forall>\<^sub>F x in finite_subsets_at_top S. y < sum f x\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  2007
      unfolding eventually_finite_subsets_at_top by auto
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2008
  qed auto
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2009
  then show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2010
    by (simp add: has_sum_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2011
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2012
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2013
lemma infsum_superconst_infinite_ennreal:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2014
  fixes f :: \<open>'a \<Rightarrow> ennreal\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2015
  assumes \<open>\<And>x. x \<in> S \<Longrightarrow> f x \<ge> b\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2016
  assumes \<open>b > 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2017
  assumes \<open>infinite S\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2018
  shows "infsum f S = \<infinity>"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2019
  using assms infsumI has_sum_superconst_infinite_ennreal by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2020
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2021
lemma infsum_superconst_infinite_ereal:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2022
  fixes f :: \<open>'a \<Rightarrow> ereal\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2023
  assumes geqb: \<open>\<And>x. x \<in> S \<Longrightarrow> f x \<ge> b\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2024
  assumes b: \<open>b > 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2025
  assumes \<open>infinite S\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2026
  shows "infsum f S = \<infinity>"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2027
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2028
  obtain b' where b': \<open>e2ennreal b' = b\<close> and \<open>b' > 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2029
    using b by blast
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2030
  have "0 < e2ennreal b"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2031
    using b' b
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2032
    by (metis dual_order.refl enn2ereal_e2ennreal gr_zeroI order_less_le zero_ennreal.abs_eq)
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2033
  hence *: \<open>infsum (e2ennreal \<circ> f) S = \<infinity>\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2034
    using assms b'
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2035
    by (intro infsum_superconst_infinite_ennreal[where b=b']) (auto intro!: e2ennreal_mono)
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2036
  have \<open>infsum f S = infsum (enn2ereal \<circ> (e2ennreal \<circ> f)) S\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2037
    using geqb b by (intro infsum_cong) (fastforce simp: enn2ereal_e2ennreal)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2038
  also have \<open>\<dots> = enn2ereal \<infinity>\<close>
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2039
    using * by (simp add: infsum_comm_additive_general continuous_at_enn2ereal nonneg_summable_on_complete)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2040
  also have \<open>\<dots> = \<infinity>\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2041
    by simp
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2042
  finally show ?thesis .
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2043
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2044
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2045
lemma has_sum_superconst_infinite_ereal:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2046
  fixes f :: \<open>'a \<Rightarrow> ereal\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2047
  assumes \<open>\<And>x. x \<in> S \<Longrightarrow> f x \<ge> b\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2048
  assumes \<open>b > 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2049
  assumes \<open>infinite S\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  2050
  shows "(f has_sum \<infinity>) S"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2051
  by (metis Infty_neq_0(1) assms infsum_def has_sum_infsum infsum_superconst_infinite_ereal)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2052
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2053
lemma infsum_superconst_infinite_enat:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2054
  fixes f :: \<open>'a \<Rightarrow> enat\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2055
  assumes geqb: \<open>\<And>x. x \<in> S \<Longrightarrow> f x \<ge> b\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2056
  assumes b: \<open>b > 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2057
  assumes \<open>infinite S\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2058
  shows "infsum f S = \<infinity>"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2059
proof -
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2060
  have \<open>ennreal_of_enat (infsum f S) = infsum (ennreal_of_enat \<circ> f) S\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2061
    by (simp flip: infsum_comm_additive_general)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2062
  also have \<open>\<dots> = \<infinity>\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2063
    by (metis assms(3) b comp_def ennreal_of_enat_0 ennreal_of_enat_le_iff geqb infsum_superconst_infinite_ennreal leD leI)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2064
  also have \<open>\<dots> = ennreal_of_enat \<infinity>\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2065
    by simp
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2066
  finally show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2067
    by (rule ennreal_of_enat_inj[THEN iffD1])
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2068
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2069
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2070
lemma has_sum_superconst_infinite_enat:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2071
  fixes f :: \<open>'a \<Rightarrow> enat\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2072
  assumes \<open>\<And>x. x \<in> S \<Longrightarrow> f x \<ge> b\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2073
  assumes \<open>b > 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2074
  assumes \<open>infinite S\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  2075
  shows "(f has_sum \<infinity>) S"
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2076
  by (metis assms i0_lb has_sum_infsum infsum_superconst_infinite_enat nonneg_summable_on_complete)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2077
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2078
text \<open>This lemma helps to relate a real-valued infsum to a supremum over extended nonnegative reals.\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2079
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2080
lemma infsum_nonneg_is_SUPREMUM_ennreal:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2081
  fixes f :: "'a \<Rightarrow> real"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2082
  assumes summable: "f summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2083
    and fnn: "\<And>x. x\<in>A \<Longrightarrow> f x \<ge> 0"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2084
  shows "ennreal (infsum f A) = (SUP F\<in>{F. finite F \<and> F \<subseteq> A}. (ennreal (sum f F)))"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2085
proof -
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2086
  have \<section>: "\<And>F. \<lbrakk>finite F; F \<subseteq> A\<rbrakk> \<Longrightarrow> sum (ennreal \<circ> f) F = ennreal (sum f F)"
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2087
    by (metis (mono_tags, lifting) comp_def fnn subsetD sum.cong sum_ennreal)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2088
  then have \<open>ennreal (infsum f A) = infsum (ennreal \<circ> f) A\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2089
    by (simp add: infsum_comm_additive_general local.summable)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2090
  also have \<open>\<dots> = (SUP F\<in>{F. finite F \<and> F \<subseteq> A}. (ennreal (sum f F)))\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2091
    by (metis (mono_tags, lifting) \<section> image_cong mem_Collect_eq nonneg_infsum_complete zero_le)
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2092
  finally show ?thesis .
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2093
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2094
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2095
text \<open>This lemma helps to related a real-valued infsum to a supremum over extended reals.\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2096
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2097
lemma infsum_nonneg_is_SUPREMUM_ereal:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2098
  fixes f :: "'a \<Rightarrow> real"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2099
  assumes summable: "f summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2100
    and fnn: "\<And>x. x\<in>A \<Longrightarrow> f x \<ge> 0"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2101
  shows "ereal (infsum f A) = (SUP F\<in>{F. finite F \<and> F \<subseteq> A}. (ereal (sum f F)))"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2102
proof -
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2103
  have "\<And>F. \<lbrakk>finite F; F \<subseteq> A\<rbrakk> \<Longrightarrow> sum (ereal \<circ> f) F = ereal (sum f F)"
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2104
    by auto
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2105
  then have \<open>ereal (infsum f A) = infsum (ereal \<circ> f) A\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2106
    by (simp add: infsum_comm_additive_general local.summable)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2107
  also have \<open>\<dots> = (SUP F\<in>{F. finite F \<and> F \<subseteq> A}. (ereal (sum f F)))\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2108
    by (subst nonneg_infsum_complete) (simp_all add: assms)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2109
  finally show ?thesis .
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2110
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2111
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2112
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2113
subsection \<open>Real numbers\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2114
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2115
text \<open>Most lemmas in the general property section already apply to real numbers.
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2116
      A few ones that are specific to reals are given here.\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2117
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2118
lemma infsum_nonneg_is_SUPREMUM_real:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2119
  fixes f :: "'a \<Rightarrow> real"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2120
  assumes summable: "f summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2121
    and fnn: "\<And>x. x\<in>A \<Longrightarrow> f x \<ge> 0"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2122
  shows "infsum f A = (SUP F\<in>{F. finite F \<and> F \<subseteq> A}. (sum f F))"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2123
proof -
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2124
  have *: "ereal (infsum f A) = (SUP F\<in>{F. finite F \<and> F \<subseteq> A}. (ereal (sum f F)))"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2125
    using assms by (rule infsum_nonneg_is_SUPREMUM_ereal)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2126
  also have "\<dots> = ereal (SUP F\<in>{F. finite F \<and> F \<subseteq> A}. (sum f F))"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2127
    by (metis (no_types, lifting) * MInfty_neq_ereal(2) PInfty_neq_ereal(2) SUP_cong abs_eq_infinity_cases ereal_SUP)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2128
  finally show ?thesis by simp
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2129
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2130
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2131
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2132
lemma has_sum_nonneg_SUPREMUM_real:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2133
  fixes f :: "'a \<Rightarrow> real"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2134
  assumes "f summable_on A" and "\<And>x. x\<in>A \<Longrightarrow> f x \<ge> 0"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  2135
  shows "(f has_sum (SUP F\<in>{F. finite F \<and> F \<subseteq> A}. (sum f F))) A"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2136
  by (metis (mono_tags, lifting) assms has_sum_infsum infsum_nonneg_is_SUPREMUM_real)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2137
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2138
lemma summable_countable_real:
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2139
  fixes f :: \<open>'a \<Rightarrow> real\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2140
  assumes \<open>f summable_on A\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2141
  shows \<open>countable {x\<in>A. f x \<noteq> 0}\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2142
  using abs_summable_countable assms summable_on_iff_abs_summable_on_real by blast
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2143
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2144
subsection \<open>Complex numbers\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2145
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2146
lemma has_sum_cnj_iff[simp]: 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2147
  fixes f :: \<open>'a \<Rightarrow> complex\<close>
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  2148
  shows \<open>((\<lambda>x. cnj (f x)) has_sum cnj a) M \<longleftrightarrow> (f has_sum a) M\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2149
  by (simp add: has_sum_def lim_cnj del: cnj_sum add: cnj_sum[symmetric, abs_def, of f])
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2150
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2151
lemma summable_on_cnj_iff[simp]:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2152
  "(\<lambda>i. cnj (f i)) summable_on A \<longleftrightarrow> f summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2153
  by (metis complex_cnj_cnj summable_on_def has_sum_cnj_iff)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2154
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2155
lemma infsum_cnj[simp]: \<open>infsum (\<lambda>x. cnj (f x)) M = cnj (infsum f M)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2156
  by (metis complex_cnj_zero infsumI has_sum_cnj_iff infsum_def summable_on_cnj_iff has_sum_infsum)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2157
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2158
lemma has_sum_Re:
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  2159
  assumes "(f has_sum a) M"
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  2160
  shows "((\<lambda>x. Re (f x)) has_sum Re a) M"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2161
  using has_sum_comm_additive[where f=Re]
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2162
  using  assms tendsto_Re by (fastforce simp add: o_def additive_def)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2163
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2164
lemma infsum_Re:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2165
  assumes "f summable_on M"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2166
  shows "infsum (\<lambda>x. Re (f x)) M = Re (infsum f M)"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2167
  by (simp add: assms has_sum_Re infsumI)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2168
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2169
lemma summable_on_Re: 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2170
  assumes "f summable_on M"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2171
  shows "(\<lambda>x. Re (f x)) summable_on M"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2172
  by (metis assms has_sum_Re summable_on_def)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2173
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2174
lemma has_sum_Im:
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  2175
  assumes "(f has_sum a) M"
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  2176
  shows "((\<lambda>x. Im (f x)) has_sum Im a) M"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2177
  using has_sum_comm_additive[where f=Im]
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2178
  using  assms tendsto_Im by (fastforce simp add: o_def additive_def)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2179
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2180
lemma infsum_Im: 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2181
  assumes "f summable_on M"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2182
  shows "infsum (\<lambda>x. Im (f x)) M = Im (infsum f M)"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2183
  by (simp add: assms has_sum_Im infsumI)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2184
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2185
lemma summable_on_Im: 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2186
  assumes "f summable_on M"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2187
  shows "(\<lambda>x. Im (f x)) summable_on M"
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2188
  by (metis assms has_sum_Im summable_on_def)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2189
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2190
lemma nonneg_infsum_le_0D_complex:
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2191
  fixes f :: "'a \<Rightarrow> complex"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2192
  assumes "infsum f A \<le> 0"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2193
    and abs_sum: "f summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2194
    and nneg: "\<And>x. x \<in> A \<Longrightarrow> f x \<ge> 0"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2195
    and "x \<in> A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2196
  shows "f x = 0"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2197
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2198
  have \<open>Im (f x) = 0\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2199
    using assms(4) less_eq_complex_def nneg by auto
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2200
  moreover have \<open>Re (f x) = 0\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2201
    using assms by (auto simp add: summable_on_Re infsum_Re less_eq_complex_def intro: nonneg_infsum_le_0D[where A=A])
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2202
  ultimately show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2203
    by (simp add: complex_eqI)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2204
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2205
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2206
lemma nonneg_has_sum_le_0D_complex:
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2207
  fixes f :: "'a \<Rightarrow> complex"
77359
bfb1acc9855e has_sum now an infix operator!!
paulson <lp15@cam.ac.uk>
parents: 77357
diff changeset
  2208
  assumes "(f has_sum a) A" and \<open>a \<le> 0\<close>
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2209
    and "\<And>x. x \<in> A \<Longrightarrow> f x \<ge> 0" and "x \<in> A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2210
  shows "f x = 0"
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2211
  by (metis assms infsumI nonneg_infsum_le_0D_complex summable_on_def)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2212
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2213
text \<open>The lemma @{thm [source] infsum_mono_neutral} above applies to various linear ordered monoids such as the reals but not to the complex numbers.
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2214
      Thus we have a separate corollary for those:\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2215
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2216
lemma infsum_mono_neutral_complex:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2217
  fixes f :: "'a \<Rightarrow> complex"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2218
  assumes [simp]: "f summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2219
    and [simp]: "g summable_on B"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2220
  assumes \<open>\<And>x. x \<in> A\<inter>B \<Longrightarrow> f x \<le> g x\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2221
  assumes \<open>\<And>x. x \<in> A-B \<Longrightarrow> f x \<le> 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2222
  assumes \<open>\<And>x. x \<in> B-A \<Longrightarrow> g x \<ge> 0\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2223
  shows \<open>infsum f A \<le> infsum g B\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2224
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2225
  have \<open>infsum (\<lambda>x. Re (f x)) A \<le> infsum (\<lambda>x. Re (g x)) B\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2226
    by (smt (verit) assms infsum_cong infsum_mono_neutral less_eq_complex_def summable_on_Re zero_complex.simps(1))
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2227
  then have Re: \<open>Re (infsum f A) \<le> Re (infsum g B)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2228
    by (metis assms(1-2) infsum_Re)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2229
  have \<open>infsum (\<lambda>x. Im (f x)) A = infsum (\<lambda>x. Im (g x)) B\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2230
    by (smt (verit, best) assms(3-5) infsum_cong_neutral less_eq_complex_def zero_complex.simps(2))
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2231
  then have Im: \<open>Im (infsum f A) = Im (infsum g B)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2232
    by (metis assms(1-2) infsum_Im)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2233
  from Re Im show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2234
    by (auto simp: less_eq_complex_def)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2235
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2236
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2237
lemma infsum_mono_complex:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2238
  \<comment> \<open>For \<^typ>\<open>real\<close>, @{thm [source] infsum_mono} can be used. 
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2239
      But \<^typ>\<open>complex\<close> does not have the right typeclass.\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2240
  fixes f g :: "'a \<Rightarrow> complex"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2241
  assumes f_sum: "f summable_on A" and g_sum: "g summable_on A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2242
  assumes leq: "\<And>x. x \<in> A \<Longrightarrow> f x \<le> g x"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2243
  shows   "infsum f A \<le> infsum g A"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2244
  by (metis DiffE IntD1 f_sum g_sum infsum_mono_neutral_complex leq)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2245
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2246
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2247
lemma infsum_nonneg_complex:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2248
  fixes f :: "'a \<Rightarrow> complex"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2249
  assumes "f summable_on M"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2250
    and "\<And>x. x \<in> M \<Longrightarrow> 0 \<le> f x"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2251
  shows "infsum f M \<ge> 0" (is "?lhs \<ge> _")
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2252
  by (metis assms infsum_0_simp summable_on_0_simp infsum_mono_complex)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2253
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2254
lemma infsum_cmod:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2255
  assumes "f summable_on M"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2256
    and fnn: "\<And>x. x \<in> M \<Longrightarrow> 0 \<le> f x"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2257
  shows "infsum (\<lambda>x. cmod (f x)) M = cmod (infsum f M)"
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2258
proof -
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2259
  have \<open>complex_of_real (infsum (\<lambda>x. cmod (f x)) M) = infsum (\<lambda>x. complex_of_real (cmod (f x))) M\<close>
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2260
  proof (rule infsum_comm_additive[symmetric, unfolded o_def])
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2261
    have "(\<lambda>z. Re (f z)) summable_on M"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2262
      using assms summable_on_Re by blast
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2263
    also have "?this \<longleftrightarrow> f abs_summable_on M"
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2264
      using fnn by (intro summable_on_cong) (auto simp: less_eq_complex_def cmod_def)
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2265
    finally show \<dots> .
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2266
  qed (auto simp: additive_def)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2267
  also have \<open>\<dots> = infsum f M\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2268
    using fnn cmod_eq_Re complex_is_Real_iff less_eq_complex_def by (force cong: infsum_cong)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2269
  finally show ?thesis
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2270
    by (metis abs_of_nonneg infsum_def le_less_trans norm_ge_zero norm_infsum_bound norm_of_real not_le order_refl)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2271
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2272
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2273
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2274
lemma summable_on_iff_abs_summable_on_complex:
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2275
  fixes f :: \<open>'a \<Rightarrow> complex\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2276
  shows \<open>f summable_on A \<longleftrightarrow> f abs_summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2277
proof (rule iffI)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2278
  assume \<open>f summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2279
  define i r ni nr n where \<open>i x = Im (f x)\<close> and \<open>r x = Re (f x)\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2280
    and \<open>ni x = norm (i x)\<close> and \<open>nr x = norm (r x)\<close> and \<open>n x = norm (f x)\<close> for x
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2281
  from \<open>f summable_on A\<close> have \<open>i summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2282
    by (simp add: i_def[abs_def] summable_on_Im)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2283
  then have [simp]: \<open>ni summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2284
    using ni_def[abs_def] summable_on_iff_abs_summable_on_real by force
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2285
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2286
  from \<open>f summable_on A\<close> have \<open>r summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2287
    by (simp add: r_def[abs_def] summable_on_Re)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2288
  then have [simp]: \<open>nr summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2289
    by (metis nr_def summable_on_cong summable_on_iff_abs_summable_on_real)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2290
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2291
  have n_sum: \<open>n x \<le> nr x + ni x\<close> for x
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2292
    by (simp add: n_def nr_def ni_def r_def i_def cmod_le)
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2293
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2294
  have *: \<open>(\<lambda>x. nr x + ni x) summable_on A\<close>
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2295
    by (simp add: summable_on_add)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2296
  have "bdd_above (sum n ` {F. F \<subseteq> A \<and> finite F})"
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2297
    apply (rule bdd_aboveI[where M=\<open>infsum (\<lambda>x. nr x + ni x) A\<close>])
76940
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2298
    using * n_sum by (auto simp flip: infsum_finite simp: ni_def nr_def intro!: infsum_mono_neutral)
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2299
  then show \<open>n summable_on A\<close>
711cef61c0ce Substantial de-applying and streamlining
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  2300
    by (simp add: n_def nonneg_bdd_above_summable_on)
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2301
next
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2302
  show \<open>f abs_summable_on A \<Longrightarrow> f summable_on A\<close>
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2303
    using abs_summable_summable by blast
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2304
qed
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2305
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2306
lemma summable_countable_complex:
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2307
  fixes f :: \<open>'a \<Rightarrow> complex\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2308
  assumes \<open>f summable_on A\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2309
  shows \<open>countable {x\<in>A. f x \<noteq> 0}\<close>
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2310
  using abs_summable_countable assms summable_on_iff_abs_summable_on_complex by blast
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2311
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2312
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2313
(* TODO: figure all this out *)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2314
inductive (in topological_space) convergent_filter :: "'a filter \<Rightarrow> bool" where
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2315
  "F \<le> nhds x \<Longrightarrow> convergent_filter F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2316
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2317
lemma (in topological_space) convergent_filter_iff: "convergent_filter F \<longleftrightarrow> (\<exists>x. F \<le> nhds x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2318
  by (auto simp: convergent_filter.simps)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2319
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2320
lemma (in uniform_space) cauchy_filter_mono:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2321
  "cauchy_filter F \<Longrightarrow> F' \<le> F \<Longrightarrow> cauchy_filter F'"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2322
  unfolding cauchy_filter_def by (meson dual_order.trans prod_filter_mono)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2323
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2324
lemma (in uniform_space) convergent_filter_cauchy: 
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2325
  assumes "convergent_filter F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2326
  shows   "cauchy_filter F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2327
  using assms cauchy_filter_mono nhds_imp_cauchy_filter[OF order.refl]
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2328
  by (auto simp: convergent_filter_iff)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2329
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2330
lemma (in topological_space) convergent_filter_bot [simp, intro]: "convergent_filter bot"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2331
  by (simp add: convergent_filter_iff)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2332
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2333
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2334
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2335
class complete_uniform_space = uniform_space +
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2336
  assumes cauchy_filter_convergent': "cauchy_filter (F :: 'a filter) \<Longrightarrow> F \<noteq> bot \<Longrightarrow> convergent_filter F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2337
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2338
lemma (in complete_uniform_space)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2339
  cauchy_filter_convergent: "cauchy_filter (F :: 'a filter) \<Longrightarrow> convergent_filter F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2340
  using cauchy_filter_convergent'[of F] by (cases "F = bot") auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2341
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2342
lemma (in complete_uniform_space) convergent_filter_iff_cauchy:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2343
  "convergent_filter F \<longleftrightarrow> cauchy_filter F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2344
  using convergent_filter_cauchy cauchy_filter_convergent by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2345
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2346
definition countably_generated_filter :: "'a filter \<Rightarrow> bool" where
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2347
  "countably_generated_filter F \<longleftrightarrow> (\<exists>U :: nat \<Rightarrow> 'a set. F = (INF (n::nat). principal (U n)))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2348
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2349
lemma countably_generated_filter_has_antimono_basis:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2350
  assumes "countably_generated_filter F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2351
  obtains B :: "nat \<Rightarrow> 'a set"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2352
  where "antimono B" and "F = (INF n. principal (B n))" and
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2353
        "\<And>P. eventually P F \<longleftrightarrow> (\<exists>i. \<forall>x\<in>B i. P x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2354
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2355
  from assms obtain B where B: "F = (INF (n::nat). principal (B n))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2356
    unfolding countably_generated_filter_def by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2358
  define B' where "B' = (\<lambda>n. \<Inter>k\<le>n. B k)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2359
  have "antimono B'"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2360
    unfolding decseq_def B'_def by force
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2361
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2362
  have "(INF n. principal (B' n)) = (INF n. INF k\<in>{..n}. principal (B k))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2363
    unfolding B'_def by (intro INF_cong refl INF_principal_finite [symmetric]) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2364
  also have "\<dots> = (INF (n::nat). principal (B n))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2365
    apply (intro antisym)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2366
    apply (meson INF_lower INF_mono atMost_iff order_refl)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2367
    apply (meson INF_greatest INF_lower UNIV_I)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2368
    done
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2369
  also have "\<dots> = F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2370
    by (simp add: B)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2371
  finally have F: "F = (INF n. principal (B' n))" ..
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2372
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2373
  moreover have "eventually P F \<longleftrightarrow> (\<exists>i. eventually P (principal (B' i)))" for P
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2374
    unfolding F using \<open>antimono B'\<close>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2375
    apply (subst eventually_INF_base)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2376
      apply (auto simp: decseq_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2377
    by (meson nat_le_linear)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2378
  ultimately show ?thesis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2379
    using \<open>antimono B'\<close> that[of B'] unfolding eventually_principal by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2380
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2381
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2382
lemma (in uniform_space) cauchy_filter_iff:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2383
  "cauchy_filter F \<longleftrightarrow> (\<forall>P. eventually P uniformity \<longrightarrow> (\<exists>X. eventually (\<lambda>x. x \<in> X) F \<and> (\<forall>z\<in>X\<times>X. P z)))" 
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2384
  unfolding cauchy_filter_def le_filter_def
79529
cb933e165dc3 tuned proof: avoid z3 to make it work on arm64-linux;
wenzelm
parents: 77388
diff changeset
  2385
  apply (auto simp: eventually_prod_same)
cb933e165dc3 tuned proof: avoid z3 to make it work on arm64-linux;
wenzelm
parents: 77388
diff changeset
  2386
   apply (metis (full_types) eventually_mono mem_Collect_eq)
cb933e165dc3 tuned proof: avoid z3 to make it work on arm64-linux;
wenzelm
parents: 77388
diff changeset
  2387
  apply blast
cb933e165dc3 tuned proof: avoid z3 to make it work on arm64-linux;
wenzelm
parents: 77388
diff changeset
  2388
  done
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2389
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2390
lemma (in uniform_space) controlled_sequences_convergent_imp_complete_aux_sequence:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2391
  fixes U :: "nat \<Rightarrow> ('a \<times> 'a) set"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2392
  fixes F :: "'a filter"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2393
  assumes "cauchy_filter F" "F \<noteq> bot"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2394
  assumes "\<And>n. eventually (\<lambda>z. z \<in> U n) uniformity"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2395
  obtains g G where
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2396
    "antimono G" "\<And>n. g n \<in> G n"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2397
    "\<And>n. eventually (\<lambda>x. x \<in> G n) F" "\<And>n. G n \<times> G n \<subseteq> U n"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2398
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2399
  have "\<exists>C. eventually (\<lambda>x. x \<in> C) F \<and> C \<times> C \<subseteq> U n" for n
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2400
    using assms(1) assms(3)[of n] unfolding cauchy_filter_iff by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2401
  then obtain G where G: "\<And>n. eventually (\<lambda>x. x \<in> G n) F" "\<And>n. G n \<times> G n \<subseteq> U n"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2402
    by metis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2403
  define G' where "G' = (\<lambda>n. \<Inter>k\<le>n. G k)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2404
  have 1: "eventually (\<lambda>x. x \<in> G' n) F" for n
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2405
    using G by (auto simp: G'_def intro: eventually_ball_finite)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2406
  have 2: "G' n \<times> G' n \<subseteq> U n" for n
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2407
    using G unfolding G'_def by fast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2408
  have 3: "antimono G'"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2409
    unfolding G'_def decseq_def by force
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2410
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2411
  have "\<exists>g. g \<in> G' n" for n
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2412
    using 1 assms(2) eventually_happens' by auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2413
  then obtain g where g: "\<And>n. g n \<in> G' n"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2414
    by metis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2415
  from g 1 2 3 that[of G' g] show ?thesis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2416
    by metis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2417
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2418
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2419
definition lift_filter :: "('a set \<Rightarrow> 'b filter) \<Rightarrow> 'a filter \<Rightarrow> 'b filter" where
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2420
  "lift_filter f F = (INF X\<in>{X. eventually (\<lambda>x. x \<in> X) F}. f X)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2421
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2422
lemma lift_filter_top [simp]: "lift_filter g top = g UNIV"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2423
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2424
  have "{X. \<forall>x::'b. x \<in> X} = {UNIV}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2425
    by auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2426
  thus ?thesis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2427
    by (simp add: lift_filter_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2428
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2429
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2430
lemma eventually_lift_filter_iff:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2431
  assumes "mono g"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2432
  shows   "eventually P (lift_filter g F) \<longleftrightarrow> (\<exists>X. eventually (\<lambda>x. x \<in> X) F \<and> eventually P (g X))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2433
  unfolding lift_filter_def
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2434
proof (subst eventually_INF_base, goal_cases)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2435
  case 1
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2436
  thus ?case by (auto intro: exI[of _ UNIV])
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2437
next
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2438
  case (2 X Y)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2439
  thus ?case
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2440
    by (auto intro!: exI[of _ "X \<inter> Y"] eventually_conj monoD[OF assms])
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2441
qed auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2442
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2443
lemma lift_filter_le:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2444
  assumes "eventually (\<lambda>x. x \<in> X) F" "g X \<le> F'"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2445
  shows   "lift_filter g F \<le> F'"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2446
  unfolding lift_filter_def
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2447
  by (metis INF_lower2 assms mem_Collect_eq)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2448
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2449
definition lift_filter' :: "('a set \<Rightarrow> 'b set) \<Rightarrow> 'a filter \<Rightarrow> 'b filter" where
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2450
  "lift_filter' f F = lift_filter (principal \<circ> f) F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2451
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2452
lemma lift_filter'_top [simp]: "lift_filter' g top = principal (g UNIV)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2453
  by (simp add: lift_filter'_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2454
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2455
lemma eventually_lift_filter'_iff:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2456
  assumes "mono g"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2457
  shows   "eventually P (lift_filter' g F) \<longleftrightarrow> (\<exists>X. eventually (\<lambda>x. x \<in> X) F \<and> (\<forall>x\<in>g X. P x))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2458
  unfolding lift_filter'_def using assms
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2459
  by (subst eventually_lift_filter_iff) (auto simp: mono_def eventually_principal)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2460
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2461
lemma lift_filter'_le:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2462
  assumes "eventually (\<lambda>x. x \<in> X) F" "principal (g X) \<le> F'"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2463
  shows   "lift_filter' g F \<le> F'"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2464
  unfolding lift_filter'_def using assms
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2465
  by (intro lift_filter_le[where X = X]) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2466
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2467
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2468
lemma (in uniform_space) comp_uniformity_le_uniformity:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2469
  "lift_filter' (\<lambda>X. X O X) uniformity \<le> uniformity"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2470
  unfolding le_filter_def
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2471
proof safe
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2472
  fix P assume P: "eventually P uniformity"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2473
  have [simp]: "mono (\<lambda>X::('a \<times> 'a) set. X O X)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2474
    by (intro monoI) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2475
  from P obtain P' where P': "eventually P' uniformity " "(\<And>x y z. P' (x, y) \<Longrightarrow> P' (y, z) \<Longrightarrow> P (x, z))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2476
    using uniformity_transE by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2477
  show "eventually P (lift_filter' (\<lambda>X. X O X) uniformity)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2478
    by (auto simp: eventually_lift_filter'_iff intro!: exI[of _ "{x. P' x}"] P')
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2479
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2480
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2481
lemma (in uniform_space) comp_mem_uniformity_sets:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2482
  assumes "eventually (\<lambda>z. z \<in> X) uniformity"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2483
  obtains Y where "eventually (\<lambda>z. z \<in> Y) uniformity" "Y O Y \<subseteq> X"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2484
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2485
  have [simp]: "mono (\<lambda>X::('a \<times> 'a) set. X O X)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2486
    by (intro monoI) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2487
  have "eventually (\<lambda>z. z \<in> X) (lift_filter' (\<lambda>X. X O X) uniformity)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2488
    using assms comp_uniformity_le_uniformity using filter_leD by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2489
  thus ?thesis using that
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2490
    by (auto simp: eventually_lift_filter'_iff)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2491
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2492
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2493
lemma (in uniform_space) le_nhds_of_cauchy_adhp_aux:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2494
  assumes "\<And>P. eventually P uniformity \<Longrightarrow> (\<exists>X. eventually (\<lambda>y. y \<in> X) F \<and> (\<forall>z\<in>X \<times> X. P z) \<and> (\<exists>y. P (x, y) \<and> y \<in> X))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2495
  shows   "F \<le> nhds x"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2496
  unfolding le_filter_def
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2497
proof safe
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2498
  fix P assume "eventually P (nhds x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2499
  hence "\<forall>\<^sub>F z in uniformity. z \<in> {z. fst z = x \<longrightarrow> P (snd z)}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2500
    by (simp add: eventually_nhds_uniformity case_prod_unfold)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2501
  then obtain Y where Y: "\<forall>\<^sub>F z in uniformity. z \<in> Y" "Y O Y \<subseteq> {z. fst z = x \<longrightarrow> P (snd z)}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2502
    using comp_mem_uniformity_sets by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2503
  obtain X y where Xy: "eventually (\<lambda>y. y \<in> X) F" "X\<times>X \<subseteq> Y" "(x, y) \<in> Y" "y \<in> X"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2504
    using assms[OF Y(1)] by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2505
  have *: "P x" if "x \<in> X" for x
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2506
    using Y(2) Xy(2-4) that unfolding relcomp_unfold by force  
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2507
  show "eventually P F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2508
    by (rule eventually_mono[OF Xy(1)]) (use * in auto)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2509
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2510
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2511
lemma (in uniform_space) eventually_uniformity_imp_nhds:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2512
  assumes "eventually P uniformity"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2513
  shows   "eventually (\<lambda>y. P (x, y)) (nhds x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2514
  using assms unfolding eventually_nhds_uniformity by (elim eventually_mono) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2515
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2516
lemma (in uniform_space) controlled_sequences_convergent_imp_complete_aux:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2517
  fixes U :: "nat \<Rightarrow> ('a \<times> 'a) set"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2518
  assumes gen: "countably_generated_filter (uniformity :: ('a \<times> 'a) filter)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2519
  assumes U: "\<And>n. eventually (\<lambda>z. z \<in> U n) uniformity"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2520
  assumes conv: "\<And>(u :: nat \<Rightarrow> 'a). (\<And>N m n. N \<le> m \<Longrightarrow> N \<le> n \<Longrightarrow> (u m, u n) \<in> U N) \<Longrightarrow> convergent u"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2521
  assumes "cauchy_filter F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2522
  shows   "convergent_filter F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2523
proof (cases "F = bot")
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2524
  case False
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2525
  note F = \<open>cauchy_filter F\<close> \<open>F \<noteq> bot\<close>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2526
  from gen obtain B :: "nat \<Rightarrow> ('a \<times> 'a) set" where B:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2527
    "antimono B" "uniformity = (INF n. principal (B n))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2528
    "\<And>P. eventually P uniformity \<longleftrightarrow> (\<exists>i. \<forall>x\<in>B i. P x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2529
    using countably_generated_filter_has_antimono_basis by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2530
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2531
  have ev_B: "eventually (\<lambda>z. z \<in> B n) uniformity" for n
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2532
    by (subst B(3)) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2533
  hence ev_B': "eventually (\<lambda>z. z \<in> B n \<inter> U n) uniformity" for n
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2534
    using U by (auto intro: eventually_conj)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2535
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2536
  obtain g G where gG: "antimono G" "\<And>n. g n \<in> G n"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2537
    "\<And>n. eventually (\<lambda>x. x \<in> G n) F" "\<And>n. G n \<times> G n \<subseteq> B n \<inter> U n"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2538
    using controlled_sequences_convergent_imp_complete_aux_sequence[of F "\<lambda>n. B n \<inter> U n", OF F ev_B']
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2539
    by metis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2540
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2541
  have "convergent g"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2542
  proof (rule conv)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2543
    fix N m n :: nat
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2544
    assume mn: "N \<le> m" "N \<le> n"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2545
    have "(g m, g n) \<in> G m \<times> G n"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2546
      using gG by auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2547
    also from mn have "\<dots> \<subseteq> G N \<times> G N"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2548
      by (intro Sigma_mono gG antimonoD[OF gG(1)])
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2549
    also have "\<dots> \<subseteq> U N"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2550
      using gG by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2551
    finally show "(g m, g n) \<in> U N" .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2552
  qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2553
  then obtain L where G: "g \<longlonglongrightarrow> L"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2554
    unfolding convergent_def by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2555
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2556
  have "F \<le> nhds L"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2557
  proof (rule le_nhds_of_cauchy_adhp_aux)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2558
    fix P :: "'a \<times> 'a \<Rightarrow> bool"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2559
    assume P: "eventually P uniformity"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2560
    hence "eventually (\<lambda>n. \<forall>x\<in>B n. P x) sequentially"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2561
      using \<open>antimono B\<close> unfolding B(3) eventually_sequentially decseq_def by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2562
    moreover have "eventually (\<lambda>n. P (L, g n)) sequentially"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2563
      using P eventually_compose_filterlim eventually_uniformity_imp_nhds G by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2564
    ultimately have "eventually (\<lambda>n. (\<forall>x\<in>B n. P x) \<and> P (L, g n)) sequentially"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2565
      by eventually_elim auto
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2566
    then obtain n where "\<forall>x\<in>B n. P x" "P (L, g n)"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2567
      unfolding eventually_at_top_linorder by blast
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2568
    then show "\<exists>X. (\<forall>\<^sub>F y in F. y \<in> X) \<and> (\<forall>z\<in>X \<times> X. P z) \<and> (\<exists>y. P (L, y) \<and> y \<in> X)"
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2569
      using gG by blast+
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2570
  qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2571
  thus "convergent_filter F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2572
    by (auto simp: convergent_filter_iff)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2573
qed auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2574
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2575
theorem (in uniform_space) controlled_sequences_convergent_imp_complete:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2576
  fixes U :: "nat \<Rightarrow> ('a \<times> 'a) set"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2577
  assumes gen: "countably_generated_filter (uniformity :: ('a \<times> 'a) filter)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2578
  assumes U: "\<And>n. eventually (\<lambda>z. z \<in> U n) uniformity"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2579
  assumes conv: "\<And>(u :: nat \<Rightarrow> 'a). (\<And>N m n. N \<le> m \<Longrightarrow> N \<le> n \<Longrightarrow> (u m, u n) \<in> U N) \<Longrightarrow> convergent u"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2580
  shows "class.complete_uniform_space open uniformity"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2581
  by unfold_locales (use assms controlled_sequences_convergent_imp_complete_aux in blast)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2582
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2583
lemma filtermap_prod_filter: "filtermap (map_prod f g) (F \<times>\<^sub>F G) = filtermap f F \<times>\<^sub>F filtermap g G"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2584
proof (intro antisym)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2585
  show "filtermap (map_prod f g) (F \<times>\<^sub>F G) \<le> filtermap f F \<times>\<^sub>F filtermap g G"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2586
    by (auto simp: le_filter_def eventually_filtermap eventually_prod_filter)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2587
next
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2588
  show "filtermap f F \<times>\<^sub>F filtermap g G \<le> filtermap (map_prod f g) (F \<times>\<^sub>F G)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2589
    unfolding le_filter_def
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2590
  proof safe
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2591
    fix P assume P: "eventually P (filtermap (map_prod f g) (F \<times>\<^sub>F G))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2592
    then obtain Pf Pg where *: "eventually Pf F" "eventually Pg G" "\<forall>x. Pf x \<longrightarrow> (\<forall>y. Pg y \<longrightarrow> P (f x, g y))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2593
      by (auto simp: eventually_filtermap eventually_prod_filter)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2594
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2595
    define Pf' where "Pf' = (\<lambda>x. \<exists>y. x = f y \<and> Pf y)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2596
    define Pg' where "Pg' = (\<lambda>x. \<exists>y. x = g y \<and> Pg y)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2597
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2598
    from *(1) have "\<forall>\<^sub>F x in F. Pf' (f x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2599
      by eventually_elim (auto simp: Pf'_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2600
    moreover from *(2) have "\<forall>\<^sub>F x in G. Pg' (g x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2601
      by eventually_elim (auto simp: Pg'_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2602
    moreover have "(\<forall>x y. Pf' x \<longrightarrow> Pg' y \<longrightarrow> P (x, y))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2603
      using *(3) by (auto simp: Pf'_def Pg'_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2604
    ultimately show "eventually P (filtermap f F \<times>\<^sub>F filtermap g G)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2605
      unfolding eventually_prod_filter eventually_filtermap
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2606
      by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2607
  qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2608
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2609
      
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2610
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2611
lemma (in uniform_space) Cauchy_seq_iff_tendsto:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2612
  "Cauchy f \<longleftrightarrow> filterlim (map_prod f f) uniformity (at_top \<times>\<^sub>F at_top)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2613
  unfolding Cauchy_uniform cauchy_filter_def filterlim_def filtermap_prod_filter ..
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2614
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2615
theorem (in uniform_space) controlled_seq_imp_Cauchy_seq:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2616
  fixes U :: "nat \<Rightarrow> ('a \<times> 'a) set"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2617
  assumes U: "\<And>P. eventually P uniformity \<Longrightarrow> (\<exists>n. \<forall>x\<in>U n. P x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2618
  assumes controlled: "\<And>N m n. N \<le> m \<Longrightarrow> N \<le> n \<Longrightarrow> (f m, f n) \<in> U N"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2619
  shows   "Cauchy f"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2620
  unfolding Cauchy_seq_iff_tendsto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2621
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2622
  show "filterlim (map_prod f f) uniformity (sequentially \<times>\<^sub>F sequentially)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2623
    unfolding filterlim_def le_filter_def
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2624
  proof safe
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2625
    fix P :: "'a \<times> 'a \<Rightarrow> bool"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2626
    assume P: "eventually P uniformity"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2627
    from U[OF this] obtain N where "\<forall>x\<in>U N. P x"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2628
      by blast
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2629
    then show "eventually P (filtermap (map_prod f f) (sequentially \<times>\<^sub>F sequentially))"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2630
      unfolding eventually_filtermap eventually_prod_sequentially
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2631
      by (metis controlled map_prod_simp)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2632
  qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2633
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2634
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2635
lemma (in uniform_space) Cauchy_seq_convergent_imp_complete_aux:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2636
  fixes U :: "nat \<Rightarrow> ('a \<times> 'a) set"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2637
  assumes gen: "countably_generated_filter (uniformity :: ('a \<times> 'a) filter)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2638
  assumes conv: "\<And>(u :: nat \<Rightarrow> 'a). Cauchy u \<Longrightarrow> convergent u"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2639
  assumes "cauchy_filter F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2640
  shows   "convergent_filter F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2641
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2642
  from gen obtain B :: "nat \<Rightarrow> ('a \<times> 'a) set" where B:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2643
    "antimono B" "uniformity = (INF n. principal (B n))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2644
    "\<And>P. eventually P uniformity \<longleftrightarrow> (\<exists>i. \<forall>x\<in>B i. P x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2645
    using countably_generated_filter_has_antimono_basis by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2646
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2647
  show ?thesis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2648
  proof (rule controlled_sequences_convergent_imp_complete_aux[where U = B])
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2649
    show "\<forall>\<^sub>F z in uniformity. z \<in> B n" for n
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2650
      unfolding B(3) by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2651
  next
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2652
    fix f :: "nat \<Rightarrow> 'a"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2653
    assume f: "\<And>N m n. N \<le> m \<Longrightarrow> N \<le> n \<Longrightarrow> (f m, f n) \<in> B N"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2654
    have "Cauchy f" using f B
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2655
      by (intro controlled_seq_imp_Cauchy_seq[where U = B]) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2656
    with conv show "convergent f"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2657
      by simp
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2658
  qed fact+
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2659
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2660
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2661
theorem (in uniform_space) Cauchy_seq_convergent_imp_complete:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2662
  fixes U :: "nat \<Rightarrow> ('a \<times> 'a) set"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2663
  assumes gen: "countably_generated_filter (uniformity :: ('a \<times> 'a) filter)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2664
  assumes conv: "\<And>(u :: nat \<Rightarrow> 'a). Cauchy u \<Longrightarrow> convergent u"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2665
  shows   "class.complete_uniform_space open uniformity"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2666
  by unfold_locales (use assms Cauchy_seq_convergent_imp_complete_aux in blast)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2667
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2668
lemma (in metric_space) countably_generated_uniformity:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2669
  "countably_generated_filter uniformity"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2670
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2671
  have "(INF e\<in>{0<..}. principal {(x, y). dist (x::'a) y < e}) =
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2672
        (INF n\<in>UNIV. principal {(x, y). dist x y < 1 / real (Suc n)})" (is "?F = ?G")
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2673
    unfolding uniformity_dist
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2674
  proof (intro antisym)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2675
    have "?G = (INF e\<in>(\<lambda>n. 1 / real (Suc n)) ` UNIV. principal {(x, y). dist x y < e})"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2676
      by (simp add: image_image)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2677
    also have "\<dots> \<ge> ?F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2678
      by (intro INF_superset_mono) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2679
    finally show "?F \<le> ?G" .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2680
  next
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2681
    show "?G \<le> ?F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2682
      unfolding le_filter_def
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2683
    proof safe
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2684
      fix P assume "eventually P ?F"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2685
      then obtain \<epsilon> where \<epsilon>: "\<epsilon> > 0" "eventually P (principal {(x, y). dist x y < \<epsilon>})"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2686
      proof (subst (asm) eventually_INF_base, goal_cases)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2687
        case (2 \<epsilon>1 \<epsilon>2)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2688
        thus ?case
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2689
          by (intro bexI[of _ "min \<epsilon>1 \<epsilon>2"]) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2690
      qed auto
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2691
      from \<open>\<epsilon> > 0\<close> obtain n where "1 / real (Suc n) < \<epsilon>"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2692
        using nat_approx_posE by blast
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2693
      then have "eventually P (principal {(x, y). dist x y < 1 / real (Suc n)})"
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2694
        using \<epsilon>(2) by (auto simp: eventually_principal)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2695
      thus "eventually P ?G"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2696
        by (intro eventually_INF1) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2697
    qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2698
  qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2699
  thus "countably_generated_filter uniformity"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2700
    unfolding countably_generated_filter_def uniformity_dist by fast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2701
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2702
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2703
subclass (in complete_space) complete_uniform_space
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2704
proof (rule Cauchy_seq_convergent_imp_complete)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2705
  show "convergent f" if "Cauchy f" for f
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2706
    using Cauchy_convergent that by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2707
qed (fact countably_generated_uniformity)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2708
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2709
lemma (in complete_uniform_space) complete_UNIV_cuspace [intro]: "complete UNIV"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2710
  unfolding complete_uniform using cauchy_filter_convergent
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2711
  by (auto simp: convergent_filter.simps)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2712
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2713
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2714
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2715
lemma norm_infsum_le:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2716
  assumes "(f has_sum S) X"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2717
  assumes "(g has_sum T) X"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2718
  assumes "\<And>x. x \<in> X \<Longrightarrow> norm (f x) \<le> g x"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2719
  shows   "norm S \<le> T"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2720
proof (rule tendsto_le)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2721
  show "((\<lambda>Y. norm (\<Sum>x\<in>Y. f x)) \<longlongrightarrow> norm S) (finite_subsets_at_top X)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2722
    using assms(1) unfolding has_sum_def by (intro tendsto_norm)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2723
  show "((\<lambda>Y. \<Sum>x\<in>Y. g x) \<longlongrightarrow> T) (finite_subsets_at_top X)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2724
    using assms(2) unfolding has_sum_def .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2725
  show "\<forall>\<^sub>F x in finite_subsets_at_top X. norm (sum f x) \<le> (\<Sum>x\<in>x. g x)"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2726
    by (simp add: assms(3) eventually_finite_subsets_at_top_weakI subsetD sum_norm_le)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2727
qed auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2728
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2729
(*
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2730
lemma summable_on_Sigma:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2731
  fixes A :: "'a set" and B :: "'a \<Rightarrow> 'b set"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2732
    and f :: \<open>'a \<Rightarrow> 'b \<Rightarrow> 'c::{comm_monoid_add, t2_space, uniform_space}\<close>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2733
  assumes plus_cont: \<open>uniformly_continuous_on UNIV (\<lambda>(x::'c,y). x+y)\<close>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2734
  assumes summableAB: "(\<lambda>(x,y). f x y) summable_on (Sigma A B)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2735
  assumes summableB: \<open>\<And>x. x\<in>A \<Longrightarrow> (f x) summable_on (B x)\<close>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2736
  shows \<open>(\<lambda>x. infsum (f x) (B x)) summable_on A\<close>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2737
*)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2738
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2739
lemma has_sum_imp_summable: "(f has_sum S) A \<Longrightarrow> f summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2740
  by (auto simp: summable_on_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2741
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2742
lemma has_sum_reindex_bij_betw:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2743
  assumes "bij_betw g A B"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2744
  shows   "((\<lambda>x. f (g x)) has_sum S) A = (f has_sum S) B"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2745
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2746
  have "((\<lambda>x. f (g x)) has_sum S) A \<longleftrightarrow> (f has_sum S) (g ` A)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2747
    by (subst has_sum_reindex) (use assms in \<open>auto dest: bij_betw_imp_inj_on simp: o_def\<close>)
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2748
  then show ?thesis
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2749
    using assms bij_betw_imp_surj_on by blast 
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2750
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2751
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2752
lemma has_sum_reindex_bij_witness:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2753
  assumes "\<And>a. a \<in> S \<Longrightarrow> i (j a) = a"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2754
  assumes "\<And>a. a \<in> S \<Longrightarrow> j a \<in> T"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2755
  assumes "\<And>b. b \<in> T \<Longrightarrow> j (i b) = b"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2756
  assumes "\<And>b. b \<in> T \<Longrightarrow> i b \<in> S"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2757
  assumes "\<And>a. a \<in> S \<Longrightarrow> h (j a) = g a"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2758
  assumes "s = s'"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2759
  shows   "(g has_sum s) S = (h has_sum s') T"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2760
  by (smt (verit, del_insts) assms bij_betwI' has_sum_cong has_sum_reindex_bij_betw)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2761
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2762
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2763
lemma has_sum_homomorphism:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2764
  assumes "(f has_sum S) A" "h 0 = 0" "\<And>a b. h (a + b) = h a + h b" "continuous_on UNIV h"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2765
  shows   "((\<lambda>x. h (f x)) has_sum (h S)) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2766
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2767
  have "sum (h \<circ> f) X = h (sum f X)" for X
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2768
    by (induction X rule: infinite_finite_induct) (simp_all add: assms)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2769
  hence sum_h: "sum (h \<circ> f) = h \<circ> sum f"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2770
    by (intro ext) auto
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2771
  then have "((h \<circ> f) has_sum h S) A"
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2772
    using assms
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2773
    by (metis UNIV_I continuous_on_def has_sum_comm_additive_general o_apply)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2774
  thus ?thesis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2775
    by (simp add: o_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2776
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2777
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2778
lemma summable_on_homomorphism:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2779
  assumes "f summable_on A" "h 0 = 0" "\<And>a b. h (a + b) = h a + h b" "continuous_on UNIV h"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2780
  shows   "(\<lambda>x. h (f x)) summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2781
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2782
  from assms(1) obtain S where "(f has_sum S) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2783
    by (auto simp: summable_on_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2784
  hence "((\<lambda>x. h (f x)) has_sum h S) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2785
    by (rule has_sum_homomorphism) (use assms in auto)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2786
  thus ?thesis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2787
    by (auto simp: summable_on_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2788
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2789
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2790
lemma infsum_homomorphism_strong:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2791
  fixes h :: "'a :: {t2_space, topological_comm_monoid_add} \<Rightarrow>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2792
                'b :: {t2_space, topological_comm_monoid_add}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2793
  assumes "(\<lambda>x. h (f x)) summable_on A \<longleftrightarrow> f summable_on A"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2794
  assumes "h 0 = 0" 
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2795
  assumes "\<And>S. (f has_sum S) A \<Longrightarrow> ((\<lambda>x. h (f x)) has_sum (h S)) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2796
  shows   "infsum (\<lambda>x. h (f x)) A = h (infsum f A)"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2797
  by (metis assms has_sum_infsum infsumI infsum_not_exists)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2798
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2799
lemma has_sum_bounded_linear:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2800
  assumes "bounded_linear h" and "(f has_sum S) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2801
  shows "((\<lambda>x. h (f x)) has_sum h S) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2802
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2803
  interpret bounded_linear h by fact
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2804
  from assms(2) show ?thesis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2805
    by (rule has_sum_homomorphism) (auto simp: add intro!: continuous_on)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2806
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2807
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2808
lemma summable_on_bounded_linear:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2809
  assumes "bounded_linear h" and "f summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2810
  shows "(\<lambda>x. h (f x)) summable_on A"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2811
  by (metis assms has_sum_bounded_linear summable_on_def)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2812
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2813
lemma summable_on_bounded_linear_iff:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2814
  assumes "bounded_linear h" and "bounded_linear h'" and "\<And>x. h' (h x) = x"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2815
  shows "(\<lambda>x. h (f x)) summable_on A \<longleftrightarrow> f summable_on A"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2816
  by (metis (full_types) assms summable_on_bounded_linear summable_on_cong)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2817
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2818
lemma infsum_bounded_linear_strong:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2819
  fixes h :: "'a :: real_normed_vector \<Rightarrow> 'b :: real_normed_vector"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2820
  assumes "(\<lambda>x. h (f x)) summable_on A \<longleftrightarrow> f summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2821
  assumes "bounded_linear h"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2822
  shows   "infsum (\<lambda>x. h (f x)) A = h (infsum f A)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2823
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2824
  interpret bounded_linear h by fact
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2825
  show ?thesis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2826
    by (rule infsum_homomorphism_strong)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2827
       (insert assms, auto intro: add continuous_on has_sum_bounded_linear)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2828
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2829
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2830
lemma infsum_bounded_linear_strong':
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2831
  fixes mult :: "'c :: zero \<Rightarrow> 'a :: real_normed_vector \<Rightarrow> 'b :: real_normed_vector"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2832
  assumes "c \<noteq> 0 \<Longrightarrow> (\<lambda>x. mult c (f x)) summable_on A \<longleftrightarrow> f summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2833
  assumes "bounded_linear (mult c)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2834
  assumes [simp]: "\<And>x. mult 0 x = 0"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2835
  shows   "infsum (\<lambda>x. mult c (f x)) A = mult c (infsum f A)"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2836
  by (metis assms infsum_0 infsum_bounded_linear_strong)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2837
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2838
lemma has_sum_of_nat: "(f has_sum S) A \<Longrightarrow> ((\<lambda>x. of_nat (f x)) has_sum of_nat S) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2839
  by (erule has_sum_homomorphism) (auto intro!: continuous_intros)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2840
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2841
lemma has_sum_of_int: "(f has_sum S) A \<Longrightarrow> ((\<lambda>x. of_int (f x)) has_sum of_int S) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2842
  by (erule has_sum_homomorphism) (auto intro!: continuous_intros)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2843
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2844
lemma summable_on_of_nat: "f summable_on A \<Longrightarrow> (\<lambda>x. of_nat (f x)) summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2845
  by (erule summable_on_homomorphism) (auto intro!: continuous_intros)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2846
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2847
lemma summable_on_of_int: "f summable_on A \<Longrightarrow> (\<lambda>x. of_int (f x)) summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2848
  by (erule summable_on_homomorphism) (auto intro!: continuous_intros)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2849
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2850
lemma summable_on_discrete_iff:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2851
  fixes f :: "'a \<Rightarrow> 'b :: {discrete_topology, topological_comm_monoid_add, cancel_comm_monoid_add}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2852
  shows "f summable_on A \<longleftrightarrow> finite {x\<in>A. f x \<noteq> 0}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2853
proof
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2854
  assume *: "finite {x\<in>A. f x \<noteq> 0}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2855
  hence "f summable_on {x\<in>A. f x \<noteq> 0}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2856
    by (rule summable_on_finite)
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2857
  then show "f summable_on A"
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2858
    by (smt (verit) DiffE mem_Collect_eq summable_on_cong_neutral) 
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2859
next
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2860
  assume "f summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2861
  then obtain S where "(f has_sum S) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2862
    by (auto simp: summable_on_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2863
  hence "\<forall>\<^sub>F x in finite_subsets_at_top A. sum f x = S"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2864
    unfolding has_sum_def tendsto_discrete .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2865
  then obtain X where X: "finite X" "X \<subseteq> A" "\<And>Y. finite Y \<Longrightarrow> X \<subseteq> Y \<Longrightarrow> Y \<subseteq> A \<Longrightarrow> sum f Y = S"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2866
    unfolding eventually_finite_subsets_at_top by metis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2867
  have "{x\<in>A. f x \<noteq> 0} \<subseteq> X"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2868
  proof
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2869
    fix x assume x: "x \<in> {x\<in>A. f x \<noteq> 0}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2870
    show "x \<in> X"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2871
    proof (rule ccontr)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2872
      assume [simp]: "x \<notin> X"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2873
      have "sum f (insert x X) = S"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2874
        using X x by (intro X) auto
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2875
      then have "f x = 0"
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2876
        using X by auto
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2877
      with x show False
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2878
        by auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2879
    qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2880
  qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2881
  thus "finite {x\<in>A. f x \<noteq> 0}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2882
    using X(1) finite_subset by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2883
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2884
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2885
lemma has_sum_imp_sums: "(f has_sum S) (UNIV :: nat set) \<Longrightarrow> f sums S"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2886
  unfolding sums_def has_sum_def by (rule filterlim_compose[OF _ filterlim_lessThan_at_top])
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2887
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2888
lemma summable_on_imp_summable: "f summable_on (UNIV :: nat set) \<Longrightarrow> summable f"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2889
  unfolding summable_on_def summable_def by (auto dest: has_sum_imp_sums)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2890
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2891
lemma summable_on_UNIV_nonneg_real_iff:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2892
  assumes "\<And>n. f n \<ge> (0 :: real)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2893
  shows   "f summable_on UNIV \<longleftrightarrow> summable f"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2894
  using assms by (auto intro: norm_summable_imp_summable_on summable_on_imp_summable)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2895
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2896
lemma summable_on_imp_bounded_partial_sums:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2897
  fixes f :: "_ \<Rightarrow> 'a :: {topological_comm_monoid_add, linorder_topology}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2898
  assumes f: "f summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2899
  shows   "\<exists>C. eventually (\<lambda>X. sum f X \<le> C) (finite_subsets_at_top A)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2900
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2901
  from assms obtain S where S: "(sum f \<longlongrightarrow> S) (finite_subsets_at_top A)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2902
    unfolding summable_on_def has_sum_def by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2903
  show ?thesis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2904
  proof (cases "\<exists>C. C > S")
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2905
    case True
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2906
    then obtain C where C: "C > S"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2907
      by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2908
    have "\<forall>\<^sub>F X in finite_subsets_at_top A. sum f X < C"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2909
      using S C by (rule order_tendstoD(2))
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2910
    thus ?thesis
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2911
      by (meson eventually_mono nless_le)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2912
  next
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2913
    case False thus ?thesis
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2914
      by (meson not_eventuallyD not_le_imp_less)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2915
  qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2916
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2917
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2918
lemma has_sum_mono':
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2919
  fixes S S' :: "'a :: {linorder_topology, ordered_comm_monoid_add, topological_comm_monoid_add}"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2920
  assumes f: "(f has_sum S) A" "(f has_sum S') B" 
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2921
     and AB: "A \<subseteq> B" "\<And>x. x \<in> B - A \<Longrightarrow> f x \<ge> 0"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2922
  shows   "S \<le> S'"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2923
  using AB has_sum_mono_neutral[OF f] by fastforce
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2924
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2925
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2926
context
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2927
  assumes "SORT_CONSTRAINT('a :: {topological_comm_monoid_add, order_topology,
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2928
             ordered_comm_monoid_add, conditionally_complete_linorder})"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2929
begin
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2930
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2931
text \<open>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2932
  Any family of non-negative numbers with bounded partial sums is summable, and the sum
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2933
  is simply the supremum of the partial sums.
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2934
\<close>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2935
lemma nonneg_bounded_partial_sums_imp_has_sum_SUP:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2936
  assumes nonneg: "\<And>x. x \<in> A \<Longrightarrow> f x \<ge> (0::'a)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2937
      and bound:  "eventually (\<lambda>X. sum f X \<le> C) (finite_subsets_at_top A)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2938
  shows   "(f has_sum (SUP X\<in>{X. X \<subseteq> A \<and> finite X}. sum f X)) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2939
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2940
  from bound obtain X0
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2941
    where X0: "X0 \<subseteq> A" "finite X0" "\<And>X. X0 \<subseteq> X \<Longrightarrow> X \<subseteq> A \<Longrightarrow> finite X \<Longrightarrow> sum f X \<le> C"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2942
    by (force simp: eventually_finite_subsets_at_top)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2943
  have bound': "sum f X \<le> C" if "X \<subseteq> A" "finite X" for X
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2944
  proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2945
    have "sum f X \<le> sum f (X \<union> X0)"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2946
      using that X0 assms(1) by (intro sum_mono2) auto
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2947
    also have "\<dots> \<le> C"
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2948
      by (simp add: X0 that)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2949
    finally show ?thesis .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2950
  qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2951
  hence bdd: "bdd_above (sum f ` {X. X \<subseteq> A \<and> finite X})"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2952
    by (auto simp: bdd_above_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2953
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2954
  show ?thesis unfolding has_sum_def
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2955
  proof (rule increasing_tendsto)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2956
    show "\<forall>\<^sub>F X in finite_subsets_at_top A. sum f X \<le> Sup (sum f ` {X. X \<subseteq> A \<and> finite X})"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2957
      by (intro eventually_finite_subsets_at_top_weakI cSUP_upper[OF _ bdd]) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2958
  next
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2959
    fix y assume "y < Sup (sum f ` {X. X \<subseteq> A \<and> finite X})"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2960
    then obtain X where X: "X \<subseteq> A" "finite X" "y < sum f X"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2961
      by (subst (asm) less_cSUP_iff[OF _ bdd]) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2962
    from X have "eventually (\<lambda>X'. X \<subseteq> X' \<and> X' \<subseteq> A \<and> finite X') (finite_subsets_at_top A)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2963
      by (auto simp: eventually_finite_subsets_at_top)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2964
    thus "eventually (\<lambda>X'. y < sum f X') (finite_subsets_at_top A)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2965
    proof eventually_elim
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2966
      case (elim X')
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2967
      note \<open>y < sum f X\<close>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2968
      also have "sum f X \<le> sum f X'"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2969
        using nonneg elim by (intro sum_mono2) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2970
      finally show ?case .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2971
    qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2972
  qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2973
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2974
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2975
lemma nonneg_bounded_partial_sums_imp_summable_on:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2976
  assumes nonneg: "\<And>x. x \<in> A \<Longrightarrow> f x \<ge> (0::'a)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2977
      and bound:  "eventually (\<lambda>X. sum f X \<le> C) (finite_subsets_at_top A)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2978
  shows   "f summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2979
  using nonneg_bounded_partial_sums_imp_has_sum_SUP[OF assms] by (auto simp: summable_on_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2980
74475
409ca22dee4c new notion of infinite sums in HOL-Analysis, ordering on complex numbers
eberlm <eberlm@in.tum.de>
parents:
diff changeset
  2981
end
74791
227915e07891 more material for HOL-Analysis.Infinite_Sum
Manuel Eberl <manuel@pruvisto.org>
parents: 74642
diff changeset
  2982
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2983
context
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2984
  assumes "SORT_CONSTRAINT('a :: {topological_comm_monoid_add, linorder_topology,
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2985
             ordered_comm_monoid_add, conditionally_complete_linorder})"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2986
begin
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2987
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2988
lemma summable_on_comparison_test:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2989
  assumes "f summable_on A" and "\<And>x. x \<in> A \<Longrightarrow> g x \<le> f x" and "\<And>x. x \<in> A \<Longrightarrow> (0::'a) \<le> g x"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2990
  shows   "g summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2991
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2992
  obtain C where C: "\<forall>\<^sub>F X in finite_subsets_at_top A. sum f X \<le> C"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  2993
    using assms(1) summable_on_imp_bounded_partial_sums by blast
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2994
  show ?thesis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2995
  proof (rule nonneg_bounded_partial_sums_imp_summable_on)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2996
    show "\<forall>\<^sub>F X in finite_subsets_at_top A. sum g X \<le> C"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2997
      using C assms 
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2998
      unfolding eventually_finite_subsets_at_top
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  2999
      by (smt (verit, ccfv_SIG) order_trans subsetD sum_mono)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3000
  qed (use assms in auto)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3001
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3002
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3003
end
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3004
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3005
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3006
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3007
lemma summable_on_subset:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3008
  fixes f :: "_ \<Rightarrow> 'a :: {uniform_topological_group_add, topological_comm_monoid_add, ab_group_add, complete_uniform_space}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3009
  assumes "f summable_on A" "B \<subseteq> A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3010
  shows "f summable_on B"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3011
  by (rule summable_on_subset_aux[OF _ _ assms]) (auto simp: uniformly_continuous_add)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3012
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3013
lemma summable_on_union:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3014
  fixes f :: "_ \<Rightarrow> 'a :: {uniform_topological_group_add, topological_comm_monoid_add, ab_group_add, complete_uniform_space}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3015
  assumes "f summable_on A" "f summable_on B"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3016
  shows "f summable_on (A \<union> B)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3017
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3018
  have "f summable_on (A \<union> (B - A))"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3019
    by (meson Diff_disjoint Diff_subset assms summable_on_Un_disjoint summable_on_subset)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3020
  also have "A \<union> (B - A) = A \<union> B"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3021
    by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3022
  finally show ?thesis .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3023
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3024
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3025
lemma summable_on_insert_iff:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3026
  fixes f :: "_ \<Rightarrow> 'a :: {uniform_topological_group_add, topological_comm_monoid_add, ab_group_add, complete_uniform_space}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3027
  shows "f summable_on insert x A \<longleftrightarrow> f summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3028
  using summable_on_union[of f A "{x}"] by (auto intro: summable_on_subset)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3029
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3030
lemma has_sum_finiteI: "finite A \<Longrightarrow> S = sum f A \<Longrightarrow> (f has_sum S) A"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3031
  by simp
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3032
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3033
lemma has_sum_insert:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3034
  fixes f :: "'a \<Rightarrow> 'b :: topological_comm_monoid_add"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3035
  assumes "x \<notin> A" and "(f has_sum S) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3036
  shows   "(f has_sum (f x + S)) (insert x A)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3037
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3038
  have "(f has_sum (f x + S)) ({x} \<union> A)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3039
    using assms by (intro has_sum_Un_disjoint) (auto intro: has_sum_finiteI)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3040
  thus ?thesis by simp
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3041
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3042
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3043
lemma infsum_insert:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3044
  fixes f :: "_ \<Rightarrow> 'a :: {topological_comm_monoid_add, t2_space}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3045
  assumes "f summable_on A" "a \<notin> A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3046
  shows   "infsum f (insert a A) = f a + infsum f A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3047
  by (meson assms has_sum_insert infsumI summable_iff_has_sum_infsum)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3048
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3049
lemma has_sum_SigmaD:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3050
  fixes f :: "'b \<times> 'c \<Rightarrow> 'a :: {topological_comm_monoid_add,t3_space}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3051
  assumes sum1: "(f has_sum S) (Sigma A B)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3052
  assumes sum2: "\<And>x. x \<in> A \<Longrightarrow> ((\<lambda>y. f (x, y)) has_sum g x) (B x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3053
  shows   "(g has_sum S) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3054
  unfolding has_sum_def tendsto_def eventually_finite_subsets_at_top
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3055
proof (safe, goal_cases)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3056
  case (1 X)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3057
  with nhds_closed[of S X] obtain X'
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3058
    where X': "S \<in> X'" "closed X'" "X' \<subseteq> X" "eventually (\<lambda>y. y \<in> X') (nhds S)" by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3059
  from X'(4) obtain X'' where X'': "S \<in> X''" "open X''" "X'' \<subseteq> X'"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3060
    by (auto simp: eventually_nhds)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3061
  with sum1 obtain Y :: "('b \<times> 'c) set"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3062
    where Y: "Y \<subseteq> Sigma A B" "finite Y"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3063
             "\<And>Z. Y \<subseteq> Z \<Longrightarrow> Z \<subseteq> Sigma A B \<Longrightarrow> finite Z \<Longrightarrow> sum f Z \<in> X''"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3064
    unfolding has_sum_def tendsto_def eventually_finite_subsets_at_top by force
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3065
  define Y1 :: "'b set" where "Y1 = fst ` Y"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3066
  from Y have Y1: "Y1 \<subseteq> A" by (auto simp: Y1_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3067
  define Y2 :: "'b \<Rightarrow> 'c set" where "Y2 = (\<lambda>x. {y. (x, y) \<in> Y})"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3068
  have Y2: "finite (Y2 x)" "Y2 x \<subseteq> B x" if "x \<in> A" for x
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3069
    using that Y(1,2) unfolding Y2_def
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3070
    by (force simp: image_iff intro: finite_subset[of _ "snd ` Y"])+
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3071
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3072
  show ?case
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3073
  proof (rule exI[of _ Y1], safe, goal_cases)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3074
    case (3 Z)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3075
    define H where "H = (INF x\<in>Z. filtercomap (\<lambda>p. p x) (finite_subsets_at_top (B x)))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3076
    
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3077
    have "sum g Z \<in> X'"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3078
    proof (rule Lim_in_closed_set)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3079
      show "closed X'" by fact
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3080
    next
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3081
      show "((\<lambda>B'. sum (\<lambda>x. sum (\<lambda>y. f (x, y)) (B' x)) Z) \<longlongrightarrow> sum g Z) H"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3082
        unfolding H_def
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3083
      proof (intro tendsto_sum filterlim_INF')
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3084
        fix x assume x: "x \<in> Z"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3085
        with 3 have "x \<in> A" by auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3086
        from sum2[OF this] have "(sum (\<lambda>y. f (x, y)) \<longlongrightarrow> g x) (finite_subsets_at_top (B x))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3087
          by (simp add: has_sum_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3088
        thus "((\<lambda>B'. sum (\<lambda>y. f (x, y)) (B' x)) \<longlongrightarrow> g x)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3089
                 (filtercomap (\<lambda>p. p x) (finite_subsets_at_top (B x)))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3090
          by (rule filterlim_compose[OF _ filterlim_filtercomap])
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3091
      qed auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3092
    next
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3093
      show "\<forall>\<^sub>F h in H. sum (\<lambda>x. sum (\<lambda>y. f (x, y)) (h x)) Z \<in> X'"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3094
        unfolding H_def
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3095
      proof (subst eventually_INF_finite[OF \<open>finite Z\<close>], rule exI, safe)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3096
        fix x assume x: "x \<in> Z"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3097
        hence x': "x \<in> A" using 3 by auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3098
        show "eventually (\<lambda>h. finite (h x) \<and> Y2 x \<subseteq> h x \<and> h x \<subseteq> B x)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3099
                (filtercomap (\<lambda>p. p x) (finite_subsets_at_top (B x)))" using 3 Y2[OF x']
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3100
          by (intro eventually_filtercomapI)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3101
             (auto simp: eventually_finite_subsets_at_top intro: exI[of _ "Y2 x"])
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3102
      next
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3103
        fix h
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3104
        assume *: "\<forall>x\<in>Z. finite (h x) \<and> Y2 x \<subseteq> h x \<and> h x \<subseteq> B x"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3105
        hence "sum (\<lambda>x. sum (\<lambda>y. f (x, y)) (h x)) Z = sum f (Sigma Z h)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3106
          using \<open>finite Z\<close> by (subst sum.Sigma) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3107
        also have "\<dots> \<in> X''"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3108
          using * 3 Y(1,2) by (intro Y; force simp: Y1_def Y2_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3109
        also have "X'' \<subseteq> X'" by fact
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3110
        finally show "sum (\<lambda>x. sum (\<lambda>y. f (x, y)) (h x)) Z \<in> X'" .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3111
      qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3112
    next
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3113
      have "H = (INF x\<in>SIGMA x:Z. {X. finite X \<and> X \<subseteq> B x}.
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3114
                  principal {y. finite (y (fst x)) \<and> snd x \<subseteq> y (fst x) \<and> y (fst x) \<subseteq> B (fst x)})"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3115
        unfolding H_def finite_subsets_at_top_def filtercomap_INF filtercomap_principal
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3116
        by (simp add: INF_Sigma)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3117
      also have "\<dots> \<noteq> bot"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3118
      proof (rule INF_filter_not_bot, subst INF_principal_finite, goal_cases)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3119
        case (2 X)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3120
        define H' where
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3121
          "H' = (\<Inter>x\<in>X. {y. finite (y (fst x)) \<and> snd x \<subseteq> y (fst x) \<and> y (fst x) \<subseteq> B (fst x)})"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3122
        from 2 have "(\<lambda>x. \<Union>(y,Y)\<in>X. if x = y then Y else {}) \<in> H'"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3123
          by (force split: if_splits simp: H'_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3124
        hence "H' \<noteq> {}" by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3125
        thus "principal H' \<noteq> bot" by (simp add: principal_eq_bot_iff)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3126
      qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3127
      finally show "H \<noteq> bot" .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3128
    qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3129
    also have "X' \<subseteq> X" by fact
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3130
    finally show "sum g Z \<in> X" .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3131
  qed (insert Y(1,2), auto simp: Y1_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3132
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3133
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3134
lemma has_sum_unique:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3135
  fixes f :: "_ \<Rightarrow> 'a :: {topological_comm_monoid_add, t2_space}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3136
  assumes "(f has_sum x) A" "(f has_sum y) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3137
  shows "x = y"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3138
  using assms unfolding has_sum_def using tendsto_unique finite_subsets_at_top_neq_bot by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3139
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3140
lemma has_sum_SigmaI:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3141
  fixes f :: "_ \<Rightarrow> 'a :: {topological_comm_monoid_add, t3_space}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3142
  assumes f: "\<And>x. x \<in> A \<Longrightarrow> ((\<lambda>y. f (x, y)) has_sum g x) (B x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3143
  assumes g: "(g has_sum S) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3144
  assumes summable: "f summable_on Sigma A B"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3145
  shows   "(f has_sum S) (Sigma A B)"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3146
  by (metis f g has_sum_SigmaD has_sum_infsum has_sum_unique local.summable)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3147
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3148
lemma summable_on_SigmaD1:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3149
  fixes f :: "_ \<Rightarrow> _ \<Rightarrow> 'a :: {complete_uniform_space, uniform_topological_group_add, ab_group_add, topological_comm_monoid_add}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3150
  assumes f: "(\<lambda>(x,y). f x y) summable_on Sigma A B"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3151
  assumes x: "x \<in> A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3152
  shows   "f x summable_on B x"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3153
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3154
  have "(\<lambda>(x,y). f x y) summable_on Sigma {x} B"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3155
    using f by (rule summable_on_subset) (use x in auto)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3156
  also have "?this \<longleftrightarrow> ((\<lambda>y. f x y) \<circ> snd) summable_on Sigma {x} B"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3157
    by (intro summable_on_cong) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3158
  also have "\<dots> \<longleftrightarrow> (\<lambda>y. f x y) summable_on snd ` Sigma {x} B"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3159
    by (intro summable_on_reindex [symmetric] inj_onI) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3160
  also have "snd ` Sigma {x} B = B x"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3161
    by (force simp: Sigma_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3162
  finally show ?thesis .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3163
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3164
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3165
lemma has_sum_swap:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3166
  "(f has_sum S) (A \<times> B) \<longleftrightarrow> ((\<lambda>(x,y). f (y,x)) has_sum S) (B \<times> A)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3167
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3168
  have "bij_betw (\<lambda>(x,y). (y,x)) (B \<times> A) (A \<times> B)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3169
    by (rule bij_betwI[of _ _ _ "\<lambda>(x,y). (y,x)"]) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3170
  from has_sum_reindex_bij_betw[OF this, where f = f] show ?thesis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3171
    by (simp add: case_prod_unfold)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3172
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3173
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3174
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3175
lemma summable_on_swap:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3176
  "f summable_on (A \<times> B) \<longleftrightarrow> (\<lambda>(x,y). f (y,x)) summable_on (B \<times> A)"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3177
  by (metis has_sum_swap summable_on_def)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3178
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3179
lemma has_sum_cmult_right_iff:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3180
  fixes c :: "'a :: {topological_semigroup_mult, field}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3181
  assumes "c \<noteq> 0"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3182
  shows   "((\<lambda>x. c * f x) has_sum S) A \<longleftrightarrow> (f has_sum (S / c)) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3183
  using has_sum_cmult_right[of f A "S/c" c]
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3184
        has_sum_cmult_right[of "\<lambda>x. c * f x" A S "inverse c"] assms
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3185
  by (auto simp: field_simps)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3186
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3187
lemma has_sum_cmult_left_iff:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3188
  fixes c :: "'a :: {topological_semigroup_mult, field}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3189
  assumes "c \<noteq> 0"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3190
  shows   "((\<lambda>x. f x * c) has_sum S) A \<longleftrightarrow> (f has_sum (S / c)) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3191
  by (smt (verit, best) assms has_sum_cmult_right_iff has_sum_cong mult.commute)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3192
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3193
lemma finite_nonzero_values_imp_summable_on:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3194
  assumes "finite {x\<in>X. f x \<noteq> 0}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3195
  shows   "f summable_on X"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3196
  by (smt (verit, del_insts) Diff_iff assms mem_Collect_eq summable_on_cong_neutral summable_on_finite)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3197
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3198
lemma summable_on_of_int_iff:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3199
  "(\<lambda>x::'a. of_int (f x) :: 'b :: real_normed_algebra_1) summable_on A \<longleftrightarrow> f summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3200
proof
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3201
  assume "f summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3202
  thus "(\<lambda>x. of_int (f x)) summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3203
    by (rule summable_on_homomorphism) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3204
next
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3205
  assume "(\<lambda>x. of_int (f x) :: 'b) summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3206
  then obtain S where "((\<lambda>x. of_int (f x) :: 'b) has_sum S) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3207
    by (auto simp: summable_on_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3208
  hence "(sum (\<lambda>x. of_int (f x) :: 'b) \<longlongrightarrow> S) (finite_subsets_at_top A)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3209
    unfolding has_sum_def .
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3210
  moreover have "1/2 > (0 :: real)"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3211
    by auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3212
  ultimately have "eventually (\<lambda>X. dist (sum (\<lambda>x. of_int (f x) :: 'b) X) S < 1/2)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3213
                     (finite_subsets_at_top A)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3214
    unfolding tendsto_iff by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3215
  then obtain X where X: "finite X" "X \<subseteq> A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3216
     "\<And>Y. finite Y \<Longrightarrow> X \<subseteq> Y \<Longrightarrow> Y \<subseteq> A \<Longrightarrow> dist (sum (\<lambda>x. of_int (f x)) Y) S < 1/2"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3217
    unfolding eventually_finite_subsets_at_top by metis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3218
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3219
  have "sum f Y = sum f X" if "finite Y" "X \<subseteq> Y" "Y \<subseteq> A" for Y
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3220
  proof -
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3221
    have "dist (sum (\<lambda>x. of_int (f x)) X) S < 1/2"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3222
      by (intro X) auto
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3223
    moreover have "dist (sum (\<lambda>x. of_int (f x)) Y) S < 1/2"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3224
      by (intro X that)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3225
    ultimately have "dist (sum (\<lambda>x. of_int (f x)) X) (sum (\<lambda>x. of_int (f x) :: 'b) Y) <
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3226
                       1/2 + 1/2"
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3227
      using dist_triangle_less_add by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3228
    thus ?thesis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3229
      by (simp add: dist_norm flip: of_int_sum of_int_diff)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3230
  qed
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3231
  then have "{x\<in>A. f x \<noteq> 0} \<subseteq> X"
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3232
    by (smt (verit) X finite_insert insert_iff mem_Collect_eq subset_eq sum.insert)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3233
  with \<open>finite X\<close> have "finite {x\<in>A. f x \<noteq> 0}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3234
    using finite_subset by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3235
  thus "f summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3236
    by (rule finite_nonzero_values_imp_summable_on)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3237
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3238
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3239
lemma summable_on_of_nat_iff:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3240
  "(\<lambda>x::'a. of_nat (f x) :: 'b :: real_normed_algebra_1) summable_on A \<longleftrightarrow> f summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3241
proof
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3242
  assume "f summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3243
  thus "(\<lambda>x. of_nat (f x) :: 'b) summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3244
    by (rule summable_on_homomorphism) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3245
next
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3246
  assume "(\<lambda>x. of_nat (f x) :: 'b) summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3247
  hence "(\<lambda>x. of_int (int (f x)) :: 'b) summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3248
    by simp
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3249
  also have "?this \<longleftrightarrow> (\<lambda>x. int (f x)) summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3250
    by (rule summable_on_of_int_iff)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3251
  also have "\<dots> \<longleftrightarrow> f summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3252
    by (simp add: summable_on_discrete_iff)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3253
  finally show "f summable_on A" .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3254
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3255
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3256
lemma infsum_of_nat:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3257
  "infsum (\<lambda>x::'a. of_nat (f x) :: 'b :: {real_normed_algebra_1}) A = of_nat (infsum f A)"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3258
  by (metis has_sum_infsum has_sum_of_nat infsumI infsum_def of_nat_0 summable_on_of_nat_iff)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3259
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3260
lemma infsum_of_int:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3261
  "infsum (\<lambda>x::'a. of_int (f x) :: 'b :: {real_normed_algebra_1}) A = of_int (infsum f A)"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3262
  by (metis has_sum_infsum has_sum_of_int infsumI infsum_not_exists of_int_0 summable_on_of_int_iff)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3263
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3264
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3265
lemma summable_on_SigmaI:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3266
  fixes f :: "_ \<Rightarrow> 'a :: {linorder_topology, ordered_comm_monoid_add, topological_comm_monoid_add,
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3267
                          conditionally_complete_linorder}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3268
  assumes f: "\<And>x. x \<in> A \<Longrightarrow> ((\<lambda>y. f (x, y)) has_sum g x) (B x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3269
  assumes g: "g summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3270
  assumes f_nonneg: "\<And>x y. x \<in> A \<Longrightarrow> y \<in> B x \<Longrightarrow> f (x, y) \<ge> (0 :: 'a)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3271
  shows   "f summable_on Sigma A B"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3272
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3273
  have g_nonneg: "g x \<ge> 0" if "x \<in> A" for x
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3274
    using f by (rule has_sum_nonneg) (use f_nonneg that in auto)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3275
  obtain C where C: "eventually (\<lambda>X. sum g X \<le> C) (finite_subsets_at_top A)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3276
    using summable_on_imp_bounded_partial_sums[OF g] by blast
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3277
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3278
  have sum_g_le: "sum g X \<le> C" if X: "finite X" "X \<subseteq> A" for X
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3279
  proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3280
    from C obtain X' where X':
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3281
      "finite X'" "X' \<subseteq> A" "\<And>Y. finite Y \<Longrightarrow> X' \<subseteq> Y \<Longrightarrow> Y \<subseteq> A \<Longrightarrow> sum g Y \<le> C"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3282
      unfolding eventually_finite_subsets_at_top by metis
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3283
    have "sum g X \<le> sum g (X \<union> X')"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3284
      using X X' by (intro sum_mono2 g_nonneg) auto
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3285
    also have "\<dots> \<le> C"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3286
      using X X'(1,2) by (intro X'(3)) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3287
    finally show ?thesis .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3288
  qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3289
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3290
  have "sum f Y \<le> C" if Y: "finite Y" "Y \<subseteq> Sigma A B" for Y
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3291
  proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3292
    define Y1 and Y2 where "Y1 = fst ` Y" and "Y2 = (\<lambda>x. snd ` {z\<in>Y. fst z = x})"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3293
    have Y12: "Y = Sigma Y1 Y2"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3294
      unfolding Y1_def Y2_def by force
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3295
    have [intro]: "finite Y1" "\<And>x. x \<in> Y1 \<Longrightarrow> finite (Y2 x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3296
      using Y unfolding Y1_def Y2_def by auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3297
    have Y12_subset: "Y1 \<subseteq> A" "\<And>x. Y2 x \<subseteq> B x"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3298
      using Y by (auto simp: Y1_def Y2_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3299
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3300
    have "sum f Y = sum f (Sigma Y1 Y2)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3301
      by (simp add: Y12)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3302
    also have "\<dots> = (\<Sum>x\<in>Y1. \<Sum>y\<in>Y2 x. f (x, y))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3303
      by (subst sum.Sigma) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3304
    also have "\<dots> \<le> (\<Sum>x\<in>Y1. g x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3305
    proof (rule sum_mono)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3306
      fix x assume x: "x \<in> Y1"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3307
      show "(\<Sum>y\<in>Y2 x. f (x, y)) \<le> g x"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3308
      proof (rule has_sum_mono')
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3309
        show "((\<lambda>y. f (x, y)) has_sum (\<Sum>y\<in>Y2 x. f (x, y))) (Y2 x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3310
          using x by (intro has_sum_finite) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3311
        show "((\<lambda>y. f (x, y)) has_sum g x) (B x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3312
          by (rule f) (use x Y12_subset in auto)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3313
        show "f (x, y) \<ge> 0" if "y \<in> B x - Y2 x" for y
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3314
          using x that Y12_subset by (intro f_nonneg) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3315
      qed (use Y12_subset in auto)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3316
    qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3317
    also have "\<dots> \<le> C"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3318
      using Y12_subset by (intro sum_g_le) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3319
    finally show ?thesis .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3320
  qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3321
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3322
  hence "\<forall>\<^sub>F X in finite_subsets_at_top (Sigma A B). sum f X \<le> C"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3323
    unfolding eventually_finite_subsets_at_top by auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3324
  thus ?thesis
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3325
    by (metis SigmaE f_nonneg nonneg_bounded_partial_sums_imp_summable_on)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3326
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3327
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3328
lemma summable_on_UnionI:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3329
  fixes f :: "_ \<Rightarrow> 'a :: {linorder_topology, ordered_comm_monoid_add, topological_comm_monoid_add,
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3330
                          conditionally_complete_linorder}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3331
  assumes f: "\<And>x. x \<in> A \<Longrightarrow> (f has_sum g x) (B x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3332
  assumes g: "g summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3333
  assumes f_nonneg: "\<And>x y. x \<in> A \<Longrightarrow> y \<in> B x \<Longrightarrow> f y \<ge> (0 :: 'a)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3334
  assumes disj: "disjoint_family_on B A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3335
  shows   "f summable_on (\<Union>x\<in>A. B x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3336
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3337
  have "f \<circ> snd summable_on Sigma A B"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3338
    using assms by (intro summable_on_SigmaI[where g = g]) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3339
  also have "?this \<longleftrightarrow> f summable_on (snd ` Sigma A B)" using assms
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3340
    by (subst summable_on_reindex; force simp: disjoint_family_on_def inj_on_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3341
  also have "snd ` (Sigma A B) = (\<Union>x\<in>A. B x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3342
    by force
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3343
  finally show ?thesis .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3344
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3345
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3346
lemma summable_on_SigmaD:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3347
  fixes f :: "'a \<times> 'b \<Rightarrow> 'c :: {topological_comm_monoid_add,t3_space}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3348
  assumes sum1: "f summable_on (Sigma A B)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3349
  assumes sum2: "\<And>x. x \<in> A \<Longrightarrow> (\<lambda>y. f (x, y)) summable_on (B x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3350
  shows   "(\<lambda>x. infsum (\<lambda>y. f (x, y)) (B x)) summable_on A"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3351
  using assms unfolding summable_on_def
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3352
  by (smt (verit, del_insts) assms has_sum_SigmaD has_sum_cong has_sum_infsum)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3353
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3354
lemma summable_on_UnionD:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3355
  fixes f :: "'a \<Rightarrow> 'c :: {topological_comm_monoid_add,t3_space}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3356
  assumes sum1: "f summable_on (\<Union>x\<in>A. B x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3357
  assumes sum2: "\<And>x. x \<in> A \<Longrightarrow> f summable_on (B x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3358
  assumes disj: "disjoint_family_on B A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3359
  shows   "(\<lambda>x. infsum f (B x)) summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3360
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3361
  have "(\<Union>x\<in>A. B x) = snd ` Sigma A B"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3362
    by (force simp: Sigma_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3363
  with sum1 have "f summable_on (snd ` Sigma A B)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3364
    by simp
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3365
  also have "?this \<longleftrightarrow> (f \<circ> snd) summable_on (Sigma A B)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3366
    using disj by (intro summable_on_reindex inj_onI) (force simp: disjoint_family_on_def)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3367
  finally show "(\<lambda>x. infsum f (B x)) summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3368
    using summable_on_SigmaD[of "f \<circ> snd" A B] sum2 by simp
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3369
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3370
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3371
lemma summable_on_Union_iff:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3372
  fixes f :: "_ \<Rightarrow> 'a :: {linorder_topology, ordered_comm_monoid_add, topological_comm_monoid_add,
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3373
                          conditionally_complete_linorder, t3_space}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3374
  assumes f: "\<And>x. x \<in> A \<Longrightarrow> (f has_sum g x) (B x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3375
  assumes f_nonneg: "\<And>x y. x \<in> A \<Longrightarrow> y \<in> B x \<Longrightarrow> f y \<ge> 0"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3376
  assumes disj: "disjoint_family_on B A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3377
  shows   "f summable_on (\<Union>x\<in>A. B x) \<longleftrightarrow> g summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3378
proof
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3379
  assume "g summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3380
  thus "f summable_on (\<Union>x\<in>A. B x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3381
    using summable_on_UnionI[of A f B g] assms by auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3382
next
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3383
  assume "f summable_on (\<Union>x\<in>A. B x)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3384
  hence "(\<lambda>x. infsum f (B x)) summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3385
    using assms by (intro summable_on_UnionD) (auto dest: has_sum_imp_summable)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3386
  also have "?this \<longleftrightarrow> g summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3387
    using assms by (intro summable_on_cong) (auto simp: infsumI)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3388
  finally show "g summable_on A" .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3389
qed
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3390
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3391
lemma has_sum_Sigma':
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3392
  fixes A :: "'a set" and B :: "'a \<Rightarrow> 'b set"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3393
    and f :: \<open>'a \<times> 'b \<Rightarrow> 'c::{comm_monoid_add,uniform_space,uniform_topological_group_add}\<close>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3394
  assumes summableAB: "(f has_sum a) (Sigma A B)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3395
  assumes summableB: \<open>\<And>x. x\<in>A \<Longrightarrow> ((\<lambda>y. f (x, y)) has_sum (b x)) (B x)\<close>
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3396
  shows "(b has_sum a) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3397
  by (intro has_sum_Sigma[OF _ assms] uniformly_continuous_add)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3398
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3399
lemma abs_summable_on_comparison_test':
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3400
  assumes "g summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3401
  assumes "\<And>x. x \<in> A \<Longrightarrow> norm (f x) \<le> g x"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3402
  shows   "(\<lambda>x. norm (f x)) summable_on A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3403
proof (rule Infinite_Sum.abs_summable_on_comparison_test)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3404
  have "g summable_on A \<longleftrightarrow> (\<lambda>x. norm (g x)) summable_on A"
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3405
    by (metis summable_on_iff_abs_summable_on_real)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3406
  with assms show "(\<lambda>x. norm (g x)) summable_on A" by blast
77388
dec831b200eb Simplified some proofs
paulson <lp15@cam.ac.uk>
parents: 77359
diff changeset
  3407
qed (use assms in fastforce)
77357
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3408
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3409
lemma has_sum_geometric_from_1:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3410
  fixes z :: "'a :: {real_normed_field, banach}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3411
  assumes "norm z < 1"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3412
  shows   "((\<lambda>n. z ^ n) has_sum (z / (1 - z))) {1..}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3413
proof -
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3414
  have [simp]: "z \<noteq> 1"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3415
    using assms by auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3416
  have "(\<lambda>n. z ^ Suc n) sums (1 / (1 - z) - 1)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3417
    using geometric_sums[of z] assms by (subst sums_Suc_iff) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3418
  also have "1 / (1 - z) - 1 = z / (1 - z)"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3419
    by (auto simp: field_simps)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3420
  finally have "(\<lambda>n. z ^ Suc n) sums (z / (1 - z))" .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3421
  moreover have "summable (\<lambda>n. norm (z ^ Suc n))"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3422
    using assms
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3423
    by (subst summable_Suc_iff) (auto simp: norm_power intro!: summable_geometric)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3424
  ultimately have "((\<lambda>n. z ^ Suc n) has_sum (z / (1 - z))) UNIV"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3425
    by (intro norm_summable_imp_has_sum)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3426
  also have "?this \<longleftrightarrow> ?thesis"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3427
    by (intro has_sum_reindex_bij_witness[of _ "\<lambda>n. n-1" "\<lambda>n. n+1"]) auto
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3428
  finally show ?thesis .
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3429
qed 
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3430
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3431
lemma has_sum_divide_const:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3432
  fixes f :: "'a \<Rightarrow> 'b :: {topological_semigroup_mult, field, semiring_0}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3433
  shows "(f has_sum S) A \<Longrightarrow> ((\<lambda>x. f x / c) has_sum (S / c)) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3434
  using has_sum_cmult_right[of f A S "inverse c"] by (simp add: field_simps)
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3435
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3436
lemma has_sum_uminusI:
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3437
  fixes f :: "'a \<Rightarrow> 'b :: {topological_semigroup_mult, ring_1}"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3438
  shows "(f has_sum S) A \<Longrightarrow> ((\<lambda>x. -f x) has_sum (-S)) A"
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3439
  using has_sum_cmult_right[of f A S "-1"] by simp
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3440
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3441
end
e65d8ee80811 New material contributed by Manuel
paulson <lp15@cam.ac.uk>
parents: 76999
diff changeset
  3442