src/HOL/BNF_Wellorder_Relation.thy
changeset 61799 4cf66f21b764
parent 60758 d8d85a8172b5
child 69593 3dda49e08b9d
--- a/src/HOL/BNF_Wellorder_Relation.thy	Mon Dec 07 10:23:50 2015 +0100
+++ b/src/HOL/BNF_Wellorder_Relation.thy	Mon Dec 07 10:38:04 2015 +0100
@@ -117,10 +117,10 @@
 
 text\<open>
 We define the successor {\em of a set}, and not of an element (the latter is of course
-a particular case).  Also, we define the maximum {\em of two elements}, @{text "max2"},
-and the minimum {\em of a set}, @{text "minim"} -- we chose these variants since we
+a particular case).  Also, we define the maximum {\em of two elements}, \<open>max2\<close>,
+and the minimum {\em of a set}, \<open>minim\<close> -- we chose these variants since we
 consider them the most useful for well-orders.  The minimum is defined in terms of the
-auxiliary relational operator @{text "isMinim"}.  Then, supremum and successor are
+auxiliary relational operator \<open>isMinim\<close>.  Then, supremum and successor are
 defined in terms of minimum as expected.
 The minimum is only meaningful for non-empty sets, and the successor is only
 meaningful for sets for which strict upper bounds exist.