added lemma
authornipkow
Mon, 28 Dec 2020 17:52:26 +0100
changeset 73016 8644c1efbda2
parent 73015 2d7060a3ea11
child 73017 9283e9d45060
added lemma
src/HOL/Analysis/Harmonic_Numbers.thy
--- a/src/HOL/Analysis/Harmonic_Numbers.thy	Sun Dec 27 17:53:08 2020 +0100
+++ b/src/HOL/Analysis/Harmonic_Numbers.thy	Mon Dec 28 17:52:26 2020 +0100
@@ -33,6 +33,9 @@
 lemma harm_pos: "n > 0 \<Longrightarrow> harm n > (0 :: 'a :: {real_normed_field,linordered_field})"
   unfolding harm_def by (intro sum_pos) simp_all
 
+lemma harm_mono: "m \<le> n \<Longrightarrow> harm m \<le> (harm n :: 'a :: {real_normed_field,linordered_field})"
+by(simp add: harm_def sum_mono2)
+
 lemma of_real_harm: "of_real (harm n) = harm n"
   unfolding harm_def by simp