src/HOL/Transcendental.thy
changeset 60688 01488b559910
parent 60301 ff82ba1893c8
child 60721 c1b7793c23a3
--- a/src/HOL/Transcendental.thy	Wed Jul 08 14:01:40 2015 +0200
+++ b/src/HOL/Transcendental.thy	Wed Jul 08 14:01:41 2015 +0200
@@ -3602,11 +3602,15 @@
     done
 qed
 
-lemma sin_zero_iff_int2: "sin x = 0 \<longleftrightarrow> (\<exists>n::int. x = real n * pi)"
+lemma sin_zero_iff_int2:
+  "sin x = 0 \<longleftrightarrow> (\<exists>n::int. x = real n * pi)"
   apply (simp only: sin_zero_iff_int)
   apply (safe elim!: evenE)
   apply (simp_all add: field_simps)
-  using dvd_triv_left by fastforce
+  apply (subst real_numeral(1) [symmetric])
+  apply (simp only: real_of_int_mult [symmetric] real_of_int_inject)
+  apply auto
+  done
 
 lemma cos_monotone_0_pi:
   assumes "0 \<le> y" and "y < x" and "x \<le> pi"