author | chaieb |
Mon, 25 Feb 2008 11:27:03 +0100 | |
changeset 26119 | cb9bdde1b444 |
parent 26118 | 6f94eb10adad |
child 26120 | 2dd43c63c100 |
--- a/src/HOL/Complex/NSCA.thy Mon Feb 25 11:27:02 2008 +0100 +++ b/src/HOL/Complex/NSCA.thy Mon Feb 25 11:27:03 2008 +0100 @@ -245,11 +245,6 @@ subsection {* Properties of @{term hRe}, @{term hIm} and @{term HComplex} *} -lemma abs_Re_le_cmod: "\<bar>Re x\<bar> \<le> cmod x" -by (induct x) simp - -lemma abs_Im_le_cmod: "\<bar>Im x\<bar> \<le> cmod x" -by (induct x) simp lemma abs_hRe_le_hcmod: "\<And>x. \<bar>hRe x\<bar> \<le> hcmod x" by transfer (rule abs_Re_le_cmod)