src/HOL/Multivariate_Analysis/Complex_Transcendental.thy
changeset 61560 7c985fd653c5
parent 61524 f2e51e704a96
child 61610 4f54d2759a0b
equal deleted inserted replaced
61559:313eca3fa847 61560:7c985fd653c5
     3 *)
     3 *)
     4 
     4 
     5 section \<open>Complex Transcendental Functions\<close>
     5 section \<open>Complex Transcendental Functions\<close>
     6 
     6 
     7 theory Complex_Transcendental
     7 theory Complex_Transcendental
     8 imports  "~~/src/HOL/Multivariate_Analysis/Complex_Analysis_Basics"
     8 imports Complex_Analysis_Basics
     9 begin
     9 begin
    10 
    10 
    11 lemma cmod_add_real_less:
    11 lemma cmod_add_real_less:
    12   assumes "Im z \<noteq> 0" "r\<noteq>0"
    12   assumes "Im z \<noteq> 0" "r\<noteq>0"
    13     shows "cmod (z + r) < cmod z + abs r"
    13     shows "cmod (z + r) < cmod z + abs r"