src/HOL/Probability/Distributions.thy
changeset 53077 a1b3784f8129
parent 53015 a1119cf551e8
child 56371 fb9ae0727548
--- a/src/HOL/Probability/Distributions.thy	Sun Aug 18 18:49:45 2013 +0200
+++ b/src/HOL/Probability/Distributions.thy	Sun Aug 18 19:59:19 2013 +0200
@@ -372,7 +372,7 @@
   also have "(\<integral> x. (x / measure lborel {a .. b}) * indicator {a .. b} x \<partial>lborel) = (a + b) / 2"
   proof (subst integral_FTC_atLeastAtMost)
     fix x
-    show "DERIV (\<lambda>x. x ^ 2 / (2 * measure lborel {a..b})) x :> x / measure lborel {a..b}"
+    show "DERIV (\<lambda>x. x\<^sup>2 / (2 * measure lborel {a..b})) x :> x / measure lborel {a..b}"
       using uniform_distributed_params[OF D]
       by (auto intro!: DERIV_intros)
     show "isCont (\<lambda>x. x / Sigma_Algebra.measure lborel {a..b}) x"