src/HOL/Complex.thy
changeset 61973 0c7e865fa7cb
parent 61969 e01015e49041
child 62101 26c0a70f78a3
equal deleted inserted replaced
61972:a70b89a3e02e 61973:0c7e865fa7cb
   380 lemmas has_derivative_Im [derivative_intros] = bounded_linear.has_derivative[OF bounded_linear_Im]
   380 lemmas has_derivative_Im [derivative_intros] = bounded_linear.has_derivative[OF bounded_linear_Im]
   381 lemmas sums_Re = bounded_linear.sums [OF bounded_linear_Re]
   381 lemmas sums_Re = bounded_linear.sums [OF bounded_linear_Re]
   382 lemmas sums_Im = bounded_linear.sums [OF bounded_linear_Im]
   382 lemmas sums_Im = bounded_linear.sums [OF bounded_linear_Im]
   383 
   383 
   384 lemma tendsto_Complex [tendsto_intros]:
   384 lemma tendsto_Complex [tendsto_intros]:
   385   "(f ---> a) F \<Longrightarrow> (g ---> b) F \<Longrightarrow> ((\<lambda>x. Complex (f x) (g x)) ---> Complex a b) F"
   385   "(f \<longlongrightarrow> a) F \<Longrightarrow> (g \<longlongrightarrow> b) F \<Longrightarrow> ((\<lambda>x. Complex (f x) (g x)) \<longlongrightarrow> Complex a b) F"
   386   by (auto intro!: tendsto_intros)
   386   by (auto intro!: tendsto_intros)
   387 
   387 
   388 lemma tendsto_complex_iff:
   388 lemma tendsto_complex_iff:
   389   "(f ---> x) F \<longleftrightarrow> (((\<lambda>x. Re (f x)) ---> Re x) F \<and> ((\<lambda>x. Im (f x)) ---> Im x) F)"
   389   "(f \<longlongrightarrow> x) F \<longleftrightarrow> (((\<lambda>x. Re (f x)) \<longlongrightarrow> Re x) F \<and> ((\<lambda>x. Im (f x)) \<longlongrightarrow> Im x) F)"
   390 proof safe
   390 proof safe
   391   assume "((\<lambda>x. Re (f x)) ---> Re x) F" "((\<lambda>x. Im (f x)) ---> Im x) F"
   391   assume "((\<lambda>x. Re (f x)) \<longlongrightarrow> Re x) F" "((\<lambda>x. Im (f x)) \<longlongrightarrow> Im x) F"
   392   from tendsto_Complex[OF this] show "(f ---> x) F"
   392   from tendsto_Complex[OF this] show "(f \<longlongrightarrow> x) F"
   393     unfolding complex.collapse .
   393     unfolding complex.collapse .
   394 qed (auto intro: tendsto_intros)
   394 qed (auto intro: tendsto_intros)
   395 
   395 
   396 lemma continuous_complex_iff: "continuous F f \<longleftrightarrow>
   396 lemma continuous_complex_iff: "continuous F f \<longleftrightarrow>
   397     continuous F (\<lambda>x. Re (f x)) \<and> continuous F (\<lambda>x. Im (f x))"
   397     continuous F (\<lambda>x. Re (f x)) \<and> continuous F (\<lambda>x. Im (f x))"
   528 lemmas isCont_cnj [simp] = bounded_linear.isCont [OF bounded_linear_cnj]
   528 lemmas isCont_cnj [simp] = bounded_linear.isCont [OF bounded_linear_cnj]
   529 lemmas continuous_cnj [simp, continuous_intros] = bounded_linear.continuous [OF bounded_linear_cnj]
   529 lemmas continuous_cnj [simp, continuous_intros] = bounded_linear.continuous [OF bounded_linear_cnj]
   530 lemmas continuous_on_cnj [simp, continuous_intros] = bounded_linear.continuous_on [OF bounded_linear_cnj]
   530 lemmas continuous_on_cnj [simp, continuous_intros] = bounded_linear.continuous_on [OF bounded_linear_cnj]
   531 lemmas has_derivative_cnj [simp, derivative_intros] = bounded_linear.has_derivative [OF bounded_linear_cnj]
   531 lemmas has_derivative_cnj [simp, derivative_intros] = bounded_linear.has_derivative [OF bounded_linear_cnj]
   532 
   532 
   533 lemma lim_cnj: "((\<lambda>x. cnj(f x)) ---> cnj l) F \<longleftrightarrow> (f ---> l) F"
   533 lemma lim_cnj: "((\<lambda>x. cnj(f x)) \<longlongrightarrow> cnj l) F \<longleftrightarrow> (f \<longlongrightarrow> l) F"
   534   by (simp add: tendsto_iff dist_complex_def complex_cnj_diff [symmetric] del: complex_cnj_diff)
   534   by (simp add: tendsto_iff dist_complex_def complex_cnj_diff [symmetric] del: complex_cnj_diff)
   535 
   535 
   536 lemma sums_cnj: "((\<lambda>x. cnj(f x)) sums cnj l) \<longleftrightarrow> (f sums l)"
   536 lemma sums_cnj: "((\<lambda>x. cnj(f x)) sums cnj l) \<longleftrightarrow> (f sums l)"
   537   by (simp add: sums_def lim_cnj cnj_setsum [symmetric] del: cnj_setsum)
   537   by (simp add: sums_def lim_cnj cnj_setsum [symmetric] del: cnj_setsum)
   538 
   538