# HG changeset patch # User huffman # Date 1313727811 25200 # Node ID 23a5137162ea94e6ea6b09eeeba0c9c8e7db1782 # Parent d81d09cdab9c221442f4dba0e44b86447b04d7eb remove more bounded_linear locale interpretations (cf. f0de18b62d63) diff -r d81d09cdab9c -r 23a5137162ea src/HOL/Complex.thy --- a/src/HOL/Complex.thy Thu Aug 18 19:53:03 2011 -0700 +++ b/src/HOL/Complex.thy Thu Aug 18 21:23:31 2011 -0700 @@ -339,12 +339,23 @@ subsection {* Completeness of the Complexes *} -interpretation Re: bounded_linear "Re" +lemma bounded_linear_Re: "bounded_linear Re" by (rule bounded_linear_intro [where K=1], simp_all add: complex_norm_def) -interpretation Im: bounded_linear "Im" +lemma bounded_linear_Im: "bounded_linear Im" by (rule bounded_linear_intro [where K=1], simp_all add: complex_norm_def) +lemmas tendsto_Re [tendsto_intros] = + bounded_linear.tendsto [OF bounded_linear_Re] + +lemmas tendsto_Im [tendsto_intros] = + bounded_linear.tendsto [OF bounded_linear_Im] + +lemmas isCont_Re [simp] = bounded_linear.isCont [OF bounded_linear_Re] +lemmas isCont_Im [simp] = bounded_linear.isCont [OF bounded_linear_Im] +lemmas Cauchy_Re = bounded_linear.Cauchy [OF bounded_linear_Re] +lemmas Cauchy_Im = bounded_linear.Cauchy [OF bounded_linear_Im] + lemma tendsto_Complex [tendsto_intros]: assumes "(f ---> a) net" and "(g ---> b) net" shows "((\x. Complex (f x) (g x)) ---> Complex a b) net" @@ -370,9 +381,9 @@ proof fix X :: "nat \ complex" assume X: "Cauchy X" - from Re.Cauchy [OF X] have 1: "(\n. Re (X n)) ----> lim (\n. Re (X n))" + from Cauchy_Re [OF X] have 1: "(\n. Re (X n)) ----> lim (\n. Re (X n))" by (simp add: Cauchy_convergent_iff convergent_LIMSEQ_iff) - from Im.Cauchy [OF X] have 2: "(\n. Im (X n)) ----> lim (\n. Im (X n))" + from Cauchy_Im [OF X] have 2: "(\n. Im (X n)) ----> lim (\n. Im (X n))" by (simp add: Cauchy_convergent_iff convergent_LIMSEQ_iff) have "X ----> Complex (lim (\n. Re (X n))) (lim (\n. Im (X n)))" using LIMSEQ_Complex [OF 1 2] by simp @@ -511,10 +522,16 @@ lemma complex_mod_mult_cnj: "cmod (z * cnj z) = (cmod z)\" by (simp add: norm_mult power2_eq_square) -interpretation cnj: bounded_linear "cnj" +lemma bounded_linear_cnj: "bounded_linear cnj" using complex_cnj_add complex_cnj_scaleR by (rule bounded_linear_intro [where K=1], simp) +lemmas tendsto_cnj [tendsto_intros] = + bounded_linear.tendsto [OF bounded_linear_cnj] + +lemmas isCont_cnj [simp] = + bounded_linear.isCont [OF bounded_linear_cnj] + subsection{*The Functions @{term sgn} and @{term arg}*}