src/HOL/Transcendental.thy
changeset 36970 fb3fdb4b585e
parent 36842 99745a4b9cc9
child 36974 b877866b5b00
--- a/src/HOL/Transcendental.thy	Mon May 17 08:40:17 2010 -0700
+++ b/src/HOL/Transcendental.thy	Mon May 17 08:45:46 2010 -0700
@@ -1778,7 +1778,7 @@
 lemma sin_pi_half [simp]: "sin(pi/2) = 1"
 apply (cut_tac x = "pi/2" in sin_cos_squared_add2)
 apply (cut_tac sin_gt_zero [OF pi_half_gt_zero pi_half_less_two])
-apply (simp add: power2_eq_square)
+apply (simp add: power2_eq_1_iff)
 done
 
 lemma cos_pi [simp]: "cos pi = -1"