src/HOL/Real.thy
changeset 67226 ec32cdaab97b
parent 67051 e7e54a0b9197
child 67399 eab6ce8368fa
--- a/src/HOL/Real.thy	Tue Dec 19 14:51:27 2017 +0100
+++ b/src/HOL/Real.thy	Tue Dec 19 13:58:12 2017 +0100
@@ -23,7 +23,7 @@
 
 subsection \<open>Preliminary lemmas\<close>
 
-text{*Useful in convergence arguments*}
+text\<open>Useful in convergence arguments\<close>
 lemma inverse_of_nat_le:
   fixes n::nat shows "\<lbrakk>n \<le> m; n\<noteq>0\<rbrakk> \<Longrightarrow> 1 / of_nat m \<le> (1::'a::linordered_field) / of_nat n"
   by (simp add: frac_le)