src/HOL/Analysis/Complex_Transcendental.thy
changeset 77166 0fb350e7477b
parent 77140 9a60c1759543
child 77179 6d2ca97a8f46
equal deleted inserted replaced
77140:9a60c1759543 77166:0fb350e7477b
  2294 qed
  2294 qed
  2295 
  2295 
  2296 lemma continuous_within_Arg: "z \<notin> \<real>\<^sub>\<le>\<^sub>0 \<Longrightarrow> continuous (at z within S) Arg"
  2296 lemma continuous_within_Arg: "z \<notin> \<real>\<^sub>\<le>\<^sub>0 \<Longrightarrow> continuous (at z within S) Arg"
  2297   using continuous_at_Arg continuous_at_imp_continuous_within by blast
  2297   using continuous_at_Arg continuous_at_imp_continuous_within by blast
  2298 
  2298 
  2299 
  2299 lemma Arg_Re_pos: "\<bar>Arg z\<bar> < pi / 2 \<longleftrightarrow> Re z > 0 \<or> z = 0"
       
  2300   using Arg_def Re_Ln_pos_lt by auto
       
  2301 
       
  2302 lemma Arg_Re_nonneg: "\<bar>Arg z\<bar> \<le> pi / 2 \<longleftrightarrow> Re z \<ge> 0"
       
  2303   using Re_Ln_pos_le[of z] by (cases "z = 0") (auto simp: Arg_eq_Im_Ln Arg_zero)
       
  2304 
       
  2305 lemma Arg_times:
       
  2306   assumes "Arg z + Arg w \<in> {-pi<..pi}" "z \<noteq> 0" "w \<noteq> 0"
       
  2307   shows   "Arg (z * w) = Arg z + Arg w"
       
  2308   using Arg_eq_Im_Ln Ln_times_simple assms by auto
       
  2309   
  2300 subsection\<open>The Unwinding Number and the Ln product Formula\<close>
  2310 subsection\<open>The Unwinding Number and the Ln product Formula\<close>
  2301 
  2311 
  2302 text\<open>Note that in this special case the unwinding number is -1, 0 or 1. But it's always an integer.\<close>
  2312 text\<open>Note that in this special case the unwinding number is -1, 0 or 1. But it's always an integer.\<close>
  2303 
  2313 
  2304 lemma is_Arg_exp_Im: "is_Arg (exp z) (Im z)"
  2314 lemma is_Arg_exp_Im: "is_Arg (exp z) (Im z)"