src/HOL/Transcendental.thy
changeset 61881 b4bfa62e799d
parent 61810 3c5040d5694a
child 61942 f02b26f7d39d
--- a/src/HOL/Transcendental.thy	Thu Dec 17 16:43:36 2015 +0100
+++ b/src/HOL/Transcendental.thy	Mon Dec 21 14:44:44 2015 +0100
@@ -4680,7 +4680,7 @@
   DERIV_arctan[THEN DERIV_chain2, derivative_intros]
   DERIV_arctan[THEN DERIV_chain2, unfolded has_field_derivative_def, derivative_intros]
 
-lemma filterlim_tan_at_right: "filterlim tan at_bot (at_right (- pi/2))"
+lemma filterlim_tan_at_right: "filterlim tan at_bot (at_right (- (pi/2)))"
   by (rule filterlim_at_bot_at_right[where Q="\<lambda>x. - pi/2 < x \<and> x < pi/2" and P="\<lambda>x. True" and g=arctan])
      (auto simp: arctan le_less eventually_at dist_real_def simp del: less_divide_eq_numeral1
            intro!: tan_monotone exI[of _ "pi/2"])