src/HOL/NthRoot.thy
changeset 70365 4df0628e8545
parent 68611 4bc4b5c0ccfc
child 70378 ebd108578ab1
equal deleted inserted replaced
70363:6d96ee03b62e 70365:4df0628e8545
   223 lemma real_root_divide: "root n (x / y) = root n x / root n y"
   223 lemma real_root_divide: "root n (x / y) = root n x / root n y"
   224   by (simp add: divide_inverse real_root_mult real_root_inverse)
   224   by (simp add: divide_inverse real_root_mult real_root_inverse)
   225 
   225 
   226 lemma real_root_abs: "0 < n \<Longrightarrow> root n \<bar>x\<bar> = \<bar>root n x\<bar>"
   226 lemma real_root_abs: "0 < n \<Longrightarrow> root n \<bar>x\<bar> = \<bar>root n x\<bar>"
   227   by (simp add: abs_if real_root_minus)
   227   by (simp add: abs_if real_root_minus)
       
   228 
       
   229 lemma root_abs_power: "n > 0 \<Longrightarrow> abs (root n (y ^n)) = abs y"
       
   230   using root_sgn_power [of n]
       
   231   by (metis abs_ge_zero power_abs real_root_abs real_root_power_cancel)
   228 
   232 
   229 lemma real_root_power: "0 < n \<Longrightarrow> root n (x ^ k) = root n x ^ k"
   233 lemma real_root_power: "0 < n \<Longrightarrow> root n (x ^ k) = root n x ^ k"
   230   by (induct k) (simp_all add: real_root_mult)
   234   by (induct k) (simp_all add: real_root_mult)
   231 
   235 
   232 
   236