# HG changeset patch # User huffman # Date 1166035188 -3600 # Node ID 1897fe3d72d51d7254b75fed1ab100843dbd2517 # Parent e38f0226e95655461f5d78537c03b27b5df27405 remove references to star_n diff -r e38f0226e956 -r 1897fe3d72d5 src/HOL/Complex/CLim.thy --- a/src/HOL/Complex/CLim.thy Wed Dec 13 19:05:45 2006 +0100 +++ b/src/HOL/Complex/CLim.thy Wed Dec 13 19:39:48 2006 +0100 @@ -85,14 +85,27 @@ apply (auto dest!: NSCLIM_const_eq [symmetric]) done +lemma starfun_norm: "( *f* (\x. norm (f x))) = (\x. hnorm (( *f* f) x))" +by transfer (rule refl) + +lemma starfun_Re: "( *f* (\x. Re (f x))) = (\x. hRe (( *f* f) x))" +by transfer (rule refl) + +lemma starfun_Im: "( *f* (\x. Im (f x))) = (\x. hIm (( *f* f) x))" +by transfer (rule refl) + +lemma star_of_Re [simp]: "star_of (Re x) = hRe (star_of x)" +by transfer (rule refl) + +lemma star_of_Im [simp]: "star_of (Im x) = hIm (star_of x)" +by transfer (rule refl) + +text"" (** another equivalence result **) lemma NSCLIM_NSCRLIM_iff: "(f -- x --NS> L) = ((%y. cmod(f y - L)) -- x --NS> 0)" -apply (auto simp add: NSLIM_def Infinitesimal_approx_minus [symmetric] Infinitesimal_hcmod_iff) -apply (auto dest!: spec) -apply (rule_tac [!] x = xa in star_cases) -apply (auto simp add: star_n_diff starfun hcmod mem_infmal_iff star_of_def) -done +by (simp add: NSLIM_def starfun_norm + approx_approx_zero_iff [symmetric] approx_minus_iff [symmetric]) (** much, much easier standard proof **) lemma CLIM_CRLIM_iff: "(f -- x --> L) = ((%y. cmod(f y - L)) -- x --> 0)" @@ -107,10 +120,9 @@ "(f -- a --NS> L) = ((%x. Re(f x)) -- a --NS> Re(L) & (%x. Im(f x)) -- a --NS> Im(L))" apply (auto intro: NSLIM_Re NSLIM_Im) -apply (auto simp add: NSLIM_def) -apply (auto dest!: spec) -apply (rule_tac x = x in star_cases) -apply (simp add: approx_approx_iff starfun star_of_def) +apply (auto simp add: NSLIM_def starfun_Re starfun_Im) +apply (auto dest!: spec) +apply (simp add: starfunC_approx_Re_Im_iff starfun_Re starfun_Im) done lemma LIM_CRLIM_Re_Im_iff: