src/HOL/Hyperreal/NthRoot.thy
changeset 23044 2ad82c359175
parent 23042 492514b39956
child 23046 12f35ece221f
equal deleted inserted replaced
23043:5dbfd67516a4 23044:2ad82c359175
   257 lemma DERIV_real_root:
   257 lemma DERIV_real_root:
   258   assumes n: "0 < n"
   258   assumes n: "0 < n"
   259   assumes x: "0 < x"
   259   assumes x: "0 < x"
   260   shows "DERIV (root n) x :> inverse (real n * root n x ^ (n - Suc 0))"
   260   shows "DERIV (root n) x :> inverse (real n * root n x ^ (n - Suc 0))"
   261 proof (rule DERIV_inverse_function)
   261 proof (rule DERIV_inverse_function)
   262   show "0 < x"
   262   show "0 < x" using x .
   263     using x .
   263   show "x < x + 1" by simp
   264   show "\<forall>y. \<bar>y - x\<bar> \<le> x \<longrightarrow> root n y ^ n = y"
   264   show "\<forall>y. 0 < y \<and> y < x + 1 \<longrightarrow> root n y ^ n = y"
   265     using n by simp
   265     using n by simp
   266   show "DERIV (\<lambda>x. x ^ n) (root n x) :> real n * root n x ^ (n - Suc 0)"
   266   show "DERIV (\<lambda>x. x ^ n) (root n x) :> real n * root n x ^ (n - Suc 0)"
   267     by (rule DERIV_pow)
   267     by (rule DERIV_pow)
   268   show "real n * root n x ^ (n - Suc 0) \<noteq> 0"
   268   show "real n * root n x ^ (n - Suc 0) \<noteq> 0"
   269     using n x by simp
   269     using n x by simp