repaired document;
authorwenzelm
Mon, 19 Oct 2015 23:07:17 +0200
changeset 61490 7c9c54eb9658
parent 61489 b8d375aee0df
child 61491 97261e6c1d42
repaired document;
src/FOL/IFOL.thy
src/FOL/ex/Classical.thy
src/FOL/ex/Intuitionistic.thy
--- a/src/FOL/IFOL.thy	Mon Oct 19 23:00:07 2015 +0200
+++ b/src/FOL/IFOL.thy	Mon Oct 19 23:07:17 2015 +0200
@@ -443,7 +443,7 @@
   done
 
 text \<open>
-  Useful with @{ML eresolve_tac} for proving equalties from known
+  Useful with @{ML eresolve_tac} for proving equalities from known
   equalities.
 
         a = b
@@ -457,7 +457,7 @@
     apply assumption+
   done
 
-text \<open>Dual of box_equals: for proving equalities backwards.\<close>
+text \<open>Dual of @{text box_equals}: for proving equalities backwards.\<close>
 lemma simp_equals: "\<lbrakk>a = c; b = d; c = d\<rbrakk> \<Longrightarrow> a = b"
   apply (rule trans)
    apply (rule trans)
--- a/src/FOL/ex/Classical.thy	Mon Oct 19 23:00:07 2015 +0200
+++ b/src/FOL/ex/Classical.thy	Mon Oct 19 23:07:17 2015 +0200
@@ -322,8 +322,8 @@
 
 text \<open>
   Other proofs: Can use @{text auto}, which cheats by using rewriting!
-  Deepen_tac alone requires 253 secs.  Or
-  by (mini_tac 1 THEN Deepen_tac 5 1)
+  @{text Deepen_tac} alone requires 253 secs.  Or
+  @{text \<open>by (mini_tac 1 THEN Deepen_tac 5 1)\<close>}.
 \<close>
 
 text\<open>44\<close>
--- a/src/FOL/ex/Intuitionistic.thy	Mon Oct 19 23:00:07 2015 +0200
+++ b/src/FOL/ex/Intuitionistic.thy	Mon Oct 19 23:07:17 2015 +0200
@@ -136,11 +136,11 @@
 
 subsection \<open>Intuitionistic FOL: propositional problems based on Pelletier.\<close>
 
-text\<open>\<not>\<not>1\<close>
+text\<open>@{text "\<not>\<not>"}1\<close>
 lemma "\<not> \<not> ((P \<longrightarrow> Q) \<longleftrightarrow> (\<not> Q \<longrightarrow> \<not> P))"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
-text\<open>\<not>\<not>2\<close>
+text\<open>@{text "\<not>\<not>"}2\<close>
 lemma "\<not> \<not> (\<not> \<not> P \<longleftrightarrow> P)"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
@@ -148,23 +148,23 @@
 lemma "\<not> (P \<longrightarrow> Q) \<longrightarrow> (Q \<longrightarrow> P)"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
-text\<open>\<not>\<not>4\<close>
+text\<open>@{text "\<not>\<not>"}4\<close>
 lemma "\<not> \<not> ((\<not> P \<longrightarrow> Q) \<longleftrightarrow> (\<not> Q \<longrightarrow> P))"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
-text\<open>\<not>\<not>5\<close>
-lemma "\<not>\<not>((P \<or> Q \<longrightarrow> P \<or> R) \<longrightarrow> P \<or> (Q \<longrightarrow> R))"
+text\<open>@{text "\<not>\<not>"}5\<close>
+lemma "\<not> \<not> ((P \<or> Q \<longrightarrow> P \<or> R) \<longrightarrow> P \<or> (Q \<longrightarrow> R))"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
-text\<open>\<not>\<not>6\<close>
+text\<open>@{text "\<not>\<not>"}6\<close>
 lemma "\<not> \<not> (P \<or> \<not> P)"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
-text\<open>\<not>\<not>7\<close>
+text\<open>@{text "\<not>\<not>"}7\<close>
 lemma "\<not> \<not> (P \<or> \<not> \<not> \<not> P)"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
-text\<open>\<not>\<not>8. Peirce's law\<close>
+text\<open>@{text "\<not>\<not>"}8. Peirce's law\<close>
 lemma "\<not> \<not> (((P \<longrightarrow> Q) \<longrightarrow> P) \<longrightarrow> P)"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
@@ -182,7 +182,7 @@
 lemma "P \<longleftrightarrow> P"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
-text\<open>\<not>\<not>12. Dijkstra's law\<close>
+text\<open>@{text "\<not>\<not>"}12. Dijkstra's law\<close>
 lemma "\<not> \<not> (((P \<longleftrightarrow> Q) \<longleftrightarrow> R) \<longleftrightarrow> (P \<longleftrightarrow> (Q \<longleftrightarrow> R)))"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
@@ -193,19 +193,19 @@
 lemma "P \<or> (Q \<and> R) \<longleftrightarrow> (P \<or> Q) \<and> (P \<or> R)"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
-text\<open>\<not>\<not>14\<close>
+text\<open>@{text "\<not>\<not>"}14\<close>
 lemma "\<not> \<not> ((P \<longleftrightarrow> Q) \<longleftrightarrow> ((Q \<or> \<not> P) \<and> (\<not> Q \<or> P)))"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
-text\<open>\<not>\<not>15\<close>
+text\<open>@{text "\<not>\<not>"}15\<close>
 lemma "\<not> \<not> ((P \<longrightarrow> Q) \<longleftrightarrow> (\<not> P \<or> Q))"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
-text\<open>\<not>\<not>16\<close>
+text\<open>@{text "\<not>\<not>"}16\<close>
 lemma "\<not> \<not> ((P \<longrightarrow> Q) \<or> (Q \<longrightarrow> P))"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
-text\<open>\<not>\<not>17\<close>
+text\<open>@{text "\<not>\<not>"}17\<close>
 lemma "\<not> \<not> (((P \<and> (Q \<longrightarrow> R)) \<longrightarrow> S) \<longleftrightarrow> ((\<not> P \<or> Q \<or> S) \<and> (\<not> P \<or> \<not> R \<or> S)))"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
@@ -271,11 +271,11 @@
   require quantifier duplication -- not currently available.
 \<close>
 
-text\<open>\<not>\<not>18\<close>
+text\<open>@{text "\<not>\<not>"}18\<close>
 lemma "\<not> \<not> (\<exists>y. \<forall>x. P(y) \<longrightarrow> P(x))"
   oops  -- \<open>NOT PROVED\<close>
 
-text\<open>\<not>\<not>19\<close>
+text\<open>@{text "\<not>\<not>"}19\<close>
 lemma "\<not> \<not> (\<exists>x. \<forall>y z. (P(y) \<longrightarrow> Q(z)) \<longrightarrow> (P(x) \<longrightarrow> Q(x)))"
   oops  -- \<open>NOT PROVED\<close>
 
@@ -293,7 +293,7 @@
 lemma "(\<forall>x. P \<longleftrightarrow> Q(x)) \<longrightarrow> (P \<longleftrightarrow> (\<forall>x. Q(x)))"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
-text\<open>\<not>\<not>23\<close>
+text\<open>@{text "\<not>\<not>"}23\<close>
 lemma "\<not> \<not> ((\<forall>x. P \<or> Q(x)) \<longleftrightarrow> (P \<or> (\<forall>x. Q(x))))"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
@@ -321,7 +321,7 @@
     \<longrightarrow> (\<exists>x. Q(x) \<and> P(x))"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
-text\<open>\<not>\<not>26\<close>
+text\<open>@{text "\<not>\<not>"}26\<close>
 lemma
   "(\<not> \<not> (\<exists>x. p(x)) \<longleftrightarrow> \<not> \<not> (\<exists>x. q(x))) \<and>
     (\<forall>x. \<forall>y. p(x) \<and> q(y) \<longrightarrow> (r(x) \<longleftrightarrow> s(y)))
@@ -337,7 +337,7 @@
   \<longrightarrow> (\<forall>x. M(x) \<longrightarrow> \<not> L(x))"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
-text\<open>\<not>\<not>28. AMENDED\<close>
+text\<open>@{text "\<not>\<not>"}28. AMENDED\<close>
 lemma
   "(\<forall>x. P(x) \<longrightarrow> (\<forall>x. Q(x))) \<and>
       (\<not> \<not> (\<forall>x. Q(x) \<or> R(x)) \<longrightarrow> (\<exists>x. Q(x) \<and> S(x))) \<and>
@@ -352,7 +352,7 @@
       (\<forall>x y. P(x) \<and> Q(y) \<longrightarrow> R(x) \<and> S(y)))"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
-text\<open>\<not>\<not>30\<close>
+text\<open>@{text "\<not>\<not>"}30\<close>
 lemma
   "(\<forall>x. (P(x) \<or> Q(x)) \<longrightarrow> \<not> R(x)) \<and>
       (\<forall>x. (Q(x) \<longrightarrow> \<not> S(x)) \<longrightarrow> P(x) \<and> R(x))
@@ -375,7 +375,7 @@
   \<longrightarrow> (\<forall>x. P(x) \<and> M(x) \<longrightarrow> L(x))"
   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
 
-text\<open>\<not>\<not>33\<close>
+text\<open>@{text "\<not>\<not>"}33\<close>
 lemma
   "(\<forall>x. \<not> \<not> (P(a) \<and> (P(x) \<longrightarrow> P(b)) \<longrightarrow> P(c))) \<longleftrightarrow>
     (\<forall>x. \<not> \<not> ((\<not> P(a) \<or> P(x) \<or> P(c)) \<and> (\<not> P(a) \<or> \<not> P(b) \<or> P(c))))"