diff -r 6001375db251 -r efdc6c533bd3 src/HOL/Complex.thy --- a/src/HOL/Complex.thy Sun Oct 19 12:47:34 2014 +0200 +++ b/src/HOL/Complex.thy Sun Oct 19 18:05:26 2014 +0200 @@ -732,8 +732,8 @@ hence cos: "cos d = 1" unfolding d_def cos_diff by simp moreover from cos have "sin d = 0" by (rule cos_one_sin_zero) ultimately have "d = 0" - unfolding sin_zero_iff even_mult_two_ex - by (auto simp add: numeral_2_eq_2 less_Suc_eq) + unfolding sin_zero_iff + by (auto simp add: numeral_2_eq_2 less_Suc_eq elim!: evenE) thus "a = x" unfolding d_def by simp qed (simp add: assms del: Re_sgn Im_sgn) with `z \ 0` show "arg z = x"