src/HOL/Analysis/Complex_Transcendental.thy
changeset 67443 3abf6a722518
parent 67371 2d9cf74943e1
child 67578 6a9a0f2bb9b4
equal deleted inserted replaced
67442:f075640b8868 67443:3abf6a722518
  2849   by (blast intro: isCont_o2 [OF _ isCont_Arcsin])
  2849   by (blast intro: isCont_o2 [OF _ isCont_Arcsin])
  2850 
  2850 
  2851 lemma sin_Arcsin [simp]: "sin(Arcsin z) = z"
  2851 lemma sin_Arcsin [simp]: "sin(Arcsin z) = z"
  2852 proof -
  2852 proof -
  2853   have "\<i>*z*2 + csqrt (1 - z\<^sup>2)*2 = 0 \<longleftrightarrow> (\<i>*z)*2 + csqrt (1 - z\<^sup>2)*2 = 0"
  2853   have "\<i>*z*2 + csqrt (1 - z\<^sup>2)*2 = 0 \<longleftrightarrow> (\<i>*z)*2 + csqrt (1 - z\<^sup>2)*2 = 0"
  2854     by (simp add: algebra_simps)  \<comment>\<open>Cancelling a factor of 2\<close>
  2854     by (simp add: algebra_simps)  \<comment> \<open>Cancelling a factor of 2\<close>
  2855   moreover have "... \<longleftrightarrow> (\<i>*z) + csqrt (1 - z\<^sup>2) = 0"
  2855   moreover have "... \<longleftrightarrow> (\<i>*z) + csqrt (1 - z\<^sup>2) = 0"
  2856     by (metis Arcsin_body_lemma distrib_right no_zero_divisors zero_neq_numeral)
  2856     by (metis Arcsin_body_lemma distrib_right no_zero_divisors zero_neq_numeral)
  2857   ultimately show ?thesis
  2857   ultimately show ?thesis
  2858     apply (simp add: sin_exp_eq Arcsin_def Arcsin_body_lemma exp_minus divide_simps)
  2858     apply (simp add: sin_exp_eq Arcsin_def Arcsin_body_lemma exp_minus divide_simps)
  2859     apply (simp add: algebra_simps)
  2859     apply (simp add: algebra_simps)
  3022   by (blast intro: isCont_o2 [OF _ isCont_Arccos])
  3022   by (blast intro: isCont_o2 [OF _ isCont_Arccos])
  3023 
  3023 
  3024 lemma cos_Arccos [simp]: "cos(Arccos z) = z"
  3024 lemma cos_Arccos [simp]: "cos(Arccos z) = z"
  3025 proof -
  3025 proof -
  3026   have "z*2 + \<i> * (2 * csqrt (1 - z\<^sup>2)) = 0 \<longleftrightarrow> z*2 + \<i> * csqrt (1 - z\<^sup>2)*2 = 0"
  3026   have "z*2 + \<i> * (2 * csqrt (1 - z\<^sup>2)) = 0 \<longleftrightarrow> z*2 + \<i> * csqrt (1 - z\<^sup>2)*2 = 0"
  3027     by (simp add: algebra_simps)  \<comment>\<open>Cancelling a factor of 2\<close>
  3027     by (simp add: algebra_simps)  \<comment> \<open>Cancelling a factor of 2\<close>
  3028   moreover have "... \<longleftrightarrow> z + \<i> * csqrt (1 - z\<^sup>2) = 0"
  3028   moreover have "... \<longleftrightarrow> z + \<i> * csqrt (1 - z\<^sup>2) = 0"
  3029     by (metis distrib_right mult_eq_0_iff zero_neq_numeral)
  3029     by (metis distrib_right mult_eq_0_iff zero_neq_numeral)
  3030   ultimately show ?thesis
  3030   ultimately show ?thesis
  3031     apply (simp add: cos_exp_eq Arccos_def Arccos_body_lemma exp_minus field_simps)
  3031     apply (simp add: cos_exp_eq Arccos_def Arccos_body_lemma exp_minus field_simps)
  3032     apply (simp add: power2_eq_square [symmetric])
  3032     apply (simp add: power2_eq_square [symmetric])