src/HOL/Complex.thy
changeset 44846 e9d1fcbc7d20
parent 44844 f74a4175a3a8
child 44902 9ba11d41cd1f
equal deleted inserted replaced
44844:f74a4175a3a8 44846:e9d1fcbc7d20
   744   by (simp add: arg_correct)
   744   by (simp add: arg_correct)
   745 
   745 
   746 lemma rcis_cmod_arg: "rcis (cmod z) (arg z) = z"
   746 lemma rcis_cmod_arg: "rcis (cmod z) (arg z) = z"
   747   by (cases "z = 0", simp_all add: rcis_def cis_arg sgn_div_norm of_real_def)
   747   by (cases "z = 0", simp_all add: rcis_def cis_arg sgn_div_norm of_real_def)
   748 
   748 
   749 lemma cos_arg_i_mult_zero_pos: (* TODO: delete *)
       
   750    "0 < y ==> cos (arg(Complex 0 y)) = 0"
       
   751   using cis_arg [of "Complex 0 y"] by (simp add: complex_eq_iff)
       
   752 
       
   753 lemma cos_arg_i_mult_zero_neg: (* TODO: delete *)
       
   754    "y < 0 ==> cos (arg(Complex 0 y)) = 0"
       
   755   using cis_arg [of "Complex 0 y"] by (simp add: complex_eq_iff)
       
   756 
       
   757 lemma cos_arg_i_mult_zero [simp]:
   749 lemma cos_arg_i_mult_zero [simp]:
   758      "y \<noteq> 0 ==> cos (arg(Complex 0 y)) = 0"
   750      "y \<noteq> 0 ==> cos (arg(Complex 0 y)) = 0"
   759   using cis_arg [of "Complex 0 y"] by (simp add: complex_eq_iff)
   751   using cis_arg [of "Complex 0 y"] by (simp add: complex_eq_iff)
   760 
   752 
   761 text {* Legacy theorem names *}
   753 text {* Legacy theorem names *}