src/HOL/Hyperreal/Series.thy
changeset 21404 eb85850d3eb7
parent 21141 f0b5e6254a1f
child 22719 c51667189bd3
equal deleted inserted replaced
21403:dd58f13a8eb4 21404:eb85850d3eb7
    13 imports SEQ
    13 imports SEQ
    14 begin
    14 begin
    15 
    15 
    16 definition
    16 definition
    17    sums  :: "(nat \<Rightarrow> 'a::real_normed_vector) \<Rightarrow> 'a \<Rightarrow> bool"
    17    sums  :: "(nat \<Rightarrow> 'a::real_normed_vector) \<Rightarrow> 'a \<Rightarrow> bool"
    18      (infixr "sums" 80)
    18      (infixr "sums" 80) where
    19    "f sums s = (%n. setsum f {0..<n}) ----> s"
    19    "f sums s = (%n. setsum f {0..<n}) ----> s"
    20 
    20 
    21    summable :: "(nat \<Rightarrow> 'a::real_normed_vector) \<Rightarrow> bool"
    21 definition
       
    22    summable :: "(nat \<Rightarrow> 'a::real_normed_vector) \<Rightarrow> bool" where
    22    "summable f = (\<exists>s. f sums s)"
    23    "summable f = (\<exists>s. f sums s)"
    23 
    24 
    24    suminf   :: "(nat \<Rightarrow> 'a::real_normed_vector) \<Rightarrow> 'a"
    25 definition
       
    26    suminf   :: "(nat \<Rightarrow> 'a::real_normed_vector) \<Rightarrow> 'a" where
    25    "suminf f = (THE s. f sums s)"
    27    "suminf f = (THE s. f sums s)"
    26 
    28 
    27 syntax
    29 syntax
    28   "_suminf" :: "idt \<Rightarrow> 'a \<Rightarrow> 'a" ("\<Sum>_. _" [0, 10] 10)
    30   "_suminf" :: "idt \<Rightarrow> 'a \<Rightarrow> 'a" ("\<Sum>_. _" [0, 10] 10)
    29 translations
    31 translations