src/HOL/Complex.thy
changeset 58740 cb9d84d3e7f2
parent 58709 efdc6c533bd3
child 58889 5b7a9633cfa8
--- a/src/HOL/Complex.thy	Tue Oct 21 17:23:16 2014 +0200
+++ b/src/HOL/Complex.thy	Tue Oct 21 21:10:44 2014 +0200
@@ -733,7 +733,7 @@
     moreover from cos have "sin d = 0" by (rule cos_one_sin_zero)
     ultimately have "d = 0"
       unfolding sin_zero_iff
-      by (auto simp add: numeral_2_eq_2 less_Suc_eq elim!: evenE)
+      by (auto elim!: evenE dest!: less_2_cases)
     thus "a = x" unfolding d_def by simp
   qed (simp add: assms del: Re_sgn Im_sgn)
   with `z \<noteq> 0` show "arg z = x"