src/HOL/Isar_examples/BasicLogic.thy
changeset 7480 0a0e0dbe1269
parent 7449 ebd975549ffe
child 7604 55566b9ec7d7
--- a/src/HOL/Isar_examples/BasicLogic.thy	Sat Sep 04 21:12:15 1999 +0200
+++ b/src/HOL/Isar_examples/BasicLogic.thy	Sat Sep 04 21:13:01 1999 +0200
@@ -80,7 +80,7 @@
   then; show "B & A";
   proof;
     assume A B;
-    show ??thesis; ..;
+    show ?thesis; ..;
   qed;
 qed;
 
@@ -123,8 +123,8 @@
   then; show "EX x. P(x)";
   proof (rule exE);
     fix a;
-    assume "P(f(a))" (is "P(??witness)");
-    show ??thesis; by (rule exI [of P ??witness]);
+    assume "P(f(a))" (is "P(?witness)");
+    show ?thesis; by (rule exI [of P ?witness]);
   qed;
 qed;
 
@@ -135,7 +135,7 @@
   proof;
     fix a;
     assume "P(f(a))";
-    show ??thesis; ..;
+    show ?thesis; ..;
   qed;
 qed;