src/HOL/Analysis/Harmonic_Numbers.thy
changeset 69597 ff784d5a5bfb
parent 69064 5840724b1d71
child 70113 c8deb8ba6d05
--- a/src/HOL/Analysis/Harmonic_Numbers.thy	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/Analysis/Harmonic_Numbers.thy	Sat Jan 05 17:24:33 2019 +0100
@@ -13,7 +13,7 @@
 
 text \<open>
   The definition of the Harmonic Numbers and the Euler-Mascheroni constant.
-  Also provides a reasonably accurate approximation of @{term "ln 2 :: real"}
+  Also provides a reasonably accurate approximation of \<^term>\<open>ln 2 :: real\<close>
   and the Euler-Mascheroni constant.
 \<close>
 
@@ -515,7 +515,7 @@
 
 
 text \<open>
-  Approximation of @{term "ln 2"}. The lower bound is accurate to about 0.03; the upper
+  Approximation of \<^term>\<open>ln 2\<close>. The lower bound is accurate to about 0.03; the upper
   bound is accurate to about 0.0015.
 \<close>
 lemma ln2_ge_two_thirds: "2/3 \<le> ln (2::real)"