src/HOL/Multivariate_Analysis/Derivative.thy
changeset 53077 a1b3784f8129
parent 51733 70abecafe9ac
child 53374 a14d2a854c02
--- a/src/HOL/Multivariate_Analysis/Derivative.thy	Sun Aug 18 18:49:45 2013 +0200
+++ b/src/HOL/Multivariate_Analysis/Derivative.thy	Sun Aug 18 19:59:19 2013 +0200
@@ -629,7 +629,7 @@
   then guess x .. note x=this
   show ?thesis proof(cases "f a = f b")
     case False
-    have "norm (f b - f a) * norm (f b - f a) = norm (f b - f a)^2"
+    have "norm (f b - f a) * norm (f b - f a) = (norm (f b - f a))\<^sup>2"
       by (simp add: power2_eq_square)
     also have "\<dots> = (f b - f a) \<bullet> (f b - f a)" unfolding power2_norm_eq_inner ..
     also have "\<dots> = (f b - f a) \<bullet> f' x (b - a)"