src/HOL/Library/Infinite_Set.thy
changeset 61585 a9599d3d7610
parent 60828 e9e272fa8daf
child 61762 d50b993b4fb9
--- a/src/HOL/Library/Infinite_Set.thy	Thu Nov 05 10:35:37 2015 +0100
+++ b/src/HOL/Library/Infinite_Set.thy	Thu Nov 05 10:39:49 2015 +0100
@@ -13,7 +13,7 @@
 text \<open>
   Some elementary facts about infinite sets, mostly by Stephan Merz.
   Beware! Because "infinite" merely abbreviates a negation, these
-  lemmas may not work well with @{text "blast"}.
+  lemmas may not work well with \<open>blast\<close>.
 \<close>
 
 abbreviation infinite :: "'a set \<Rightarrow> bool"
@@ -96,7 +96,7 @@
 
 text \<open>
   For a set of natural numbers to be infinite, it is enough to know
-  that for any number larger than some @{text k}, there is some larger
+  that for any number larger than some \<open>k\<close>, there is some larger
   number that is an element of the set.
 \<close>