src/HOL/NthRoot.thy
changeset 70722 ae2528273eeb
parent 70378 ebd108578ab1
child 78127 24b70433c2e8
equal deleted inserted replaced
70721:47258727fa42 70722:ae2528273eeb
   266   from assms have "root N (root n x) ^ N < root n (root N x) ^ n"
   266   from assms have "root N (root n x) ^ N < root n (root N x) ^ n"
   267     by (simp add: real_root_commute power_strict_decreasing del: real_root_pow_pos2)
   267     by (simp add: real_root_commute power_strict_decreasing del: real_root_pow_pos2)
   268   with assms show ?thesis by simp
   268   with assms show ?thesis by simp
   269 qed
   269 qed
   270 
   270 
   271 lemma real_root_decreasing: "0 < n \<Longrightarrow> n < N \<Longrightarrow> 1 \<le> x \<Longrightarrow> root N x \<le> root n x"
   271 lemma real_root_decreasing: "0 < n \<Longrightarrow> n \<le> N \<Longrightarrow> 1 \<le> x \<Longrightarrow> root N x \<le> root n x"
   272   by (auto simp add: order_le_less real_root_strict_decreasing)
   272   by (auto simp add: order_le_less real_root_strict_decreasing)
   273 
   273 
   274 lemma real_root_increasing: "0 < n \<Longrightarrow> n < N \<Longrightarrow> 0 \<le> x \<Longrightarrow> x \<le> 1 \<Longrightarrow> root n x \<le> root N x"
   274 lemma real_root_increasing: "0 < n \<Longrightarrow> n \<le> N \<Longrightarrow> 0 \<le> x \<Longrightarrow> x \<le> 1 \<Longrightarrow> root n x \<le> root N x"
   275   by (auto simp add: order_le_less real_root_strict_increasing)
   275   by (auto simp add: order_le_less real_root_strict_increasing)
   276 
   276 
   277 
   277 
   278 text \<open>Continuity and derivatives.\<close>
   278 text \<open>Continuity and derivatives.\<close>
   279 
   279