src/HOL/Transcendental.thy
changeset 60688 01488b559910
parent 60301 ff82ba1893c8
child 60721 c1b7793c23a3
equal deleted inserted replaced
60687:33dbbcb6a8a3 60688:01488b559910
  3600     apply (rule disjI2)
  3600     apply (rule disjI2)
  3601     apply (rule_tac x="nat (-n)" in exI, simp)
  3601     apply (rule_tac x="nat (-n)" in exI, simp)
  3602     done
  3602     done
  3603 qed
  3603 qed
  3604 
  3604 
  3605 lemma sin_zero_iff_int2: "sin x = 0 \<longleftrightarrow> (\<exists>n::int. x = real n * pi)"
  3605 lemma sin_zero_iff_int2:
       
  3606   "sin x = 0 \<longleftrightarrow> (\<exists>n::int. x = real n * pi)"
  3606   apply (simp only: sin_zero_iff_int)
  3607   apply (simp only: sin_zero_iff_int)
  3607   apply (safe elim!: evenE)
  3608   apply (safe elim!: evenE)
  3608   apply (simp_all add: field_simps)
  3609   apply (simp_all add: field_simps)
  3609   using dvd_triv_left by fastforce
  3610   apply (subst real_numeral(1) [symmetric])
       
  3611   apply (simp only: real_of_int_mult [symmetric] real_of_int_inject)
       
  3612   apply auto
       
  3613   done
  3610 
  3614 
  3611 lemma cos_monotone_0_pi:
  3615 lemma cos_monotone_0_pi:
  3612   assumes "0 \<le> y" and "y < x" and "x \<le> pi"
  3616   assumes "0 \<le> y" and "y < x" and "x \<le> pi"
  3613   shows "cos x < cos y"
  3617   shows "cos x < cos y"
  3614 proof -
  3618 proof -