src/FOL/IFOL.thy
changeset 63906 fa799a8e4adc
parent 63901 4ce989e962e0
child 68816 5a53724fe247
--- a/src/FOL/IFOL.thy	Fri Sep 16 12:30:55 2016 +0200
+++ b/src/FOL/IFOL.thy	Sat Sep 17 11:41:13 2016 +0200
@@ -275,10 +275,10 @@
 text \<open>
   NOTE THAT the following 2 quantifications:
 
-    \<^item> \<exists>!x such that [\<exists>!y such that P(x,y)]     (sequential)
-    \<^item> \<exists>!x,y such that P(x,y)                   (simultaneous)
+    \<^item> \<open>\<exists>!x\<close> such that [\<open>\<exists>!y\<close> such that P(x,y)]   (sequential)
+    \<^item> \<open>\<exists>!x,y\<close> such that P(x,y)                   (simultaneous)
 
-  do NOT mean the same thing. The parser treats \<exists>!x y.P(x,y) as sequential.
+  do NOT mean the same thing. The parser treats \<open>\<exists>!x y.P(x,y)\<close> as sequential.
 \<close>
 
 lemma ex1I: "P(a) \<Longrightarrow> (\<And>x. P(x) \<Longrightarrow> x = a) \<Longrightarrow> \<exists>!x. P(x)"