src/HOL/Transcendental.thy
changeset 67727 ce3e87a51488
parent 67685 bdff8bf0a75b
child 68077 ee8c13ae81e9
--- a/src/HOL/Transcendental.thy	Sun Feb 25 20:05:05 2018 +0100
+++ b/src/HOL/Transcendental.thy	Mon Feb 26 07:34:05 2018 +0100
@@ -2910,13 +2910,8 @@
 lemma log_base_root: "n > 0 \<Longrightarrow> b > 0 \<Longrightarrow> log (root n b) x = n * (log b x)"
   by (simp add: log_def ln_root)
 
-lemma ln_bound: "1 \<le> x \<Longrightarrow> ln x \<le> x"
-  for x :: real
-  apply (subgoal_tac "ln (1 + (x - 1)) \<le> x - 1")
-   apply simp
-  apply (rule ln_add_one_self_le_self)
-  apply simp
-  done
+lemma ln_bound: "0 < x \<Longrightarrow> ln x \<le> x" for x :: real
+  using ln_le_minus_one by force
 
 lemma powr_mono: "a \<le> b \<Longrightarrow> 1 \<le> x \<Longrightarrow> x powr a \<le> x powr b"
   for x :: real