src/HOL/Analysis/Gamma_Function.thy
changeset 68224 1f7308050349
parent 68046 6aba668aea78
child 68403 223172b97d0b
equal deleted inserted replaced
68223:88dd06301dd3 68224:1f7308050349
   333 
   333 
   334 text \<open>
   334 text \<open>
   335   We now show that the log-Gamma series converges locally uniformly for all complex numbers except
   335   We now show that the log-Gamma series converges locally uniformly for all complex numbers except
   336   the non-positive integers. We do this by proving that the series is locally Cauchy, adapting this
   336   the non-positive integers. We do this by proving that the series is locally Cauchy, adapting this
   337   proof:
   337   proof:
   338   http://math.stackexchange.com/questions/887158/convergence-of-gammaz-lim-n-to-infty-fracnzn-prod-m-0nzm
   338   https://math.stackexchange.com/questions/887158/convergence-of-gammaz-lim-n-to-infty-fracnzn-prod-m-0nzm
   339 \<close>
   339 \<close>
   340 
   340 
   341 context
   341 context
   342 begin
   342 begin
   343 
   343