src/HOL/Isar_examples/Group.thy
changeset 7480 0a0e0dbe1269
parent 7433 27887c52b9c8
child 7740 2fbe5ce9845f
--- a/src/HOL/Isar_examples/Group.thy	Sat Sep 04 21:12:15 1999 +0200
+++ b/src/HOL/Isar_examples/Group.thy	Sat Sep 04 21:13:01 1999 +0200
@@ -49,7 +49,7 @@
     by (simp only: group_left_unit);
   also; have "... = one";
     by (simp only: group_left_inverse);
-  finally; show ??thesis; .;
+  finally; show ?thesis; .;
 qed;
 
 text {*
@@ -67,7 +67,7 @@
     by (simp only: group_right_inverse);
   also; have "... = x";
     by (simp only: group_left_unit);
-  finally; show ??thesis; .;
+  finally; show ?thesis; .;
 qed;
 
 text {*
@@ -80,7 +80,7 @@
 
  Note that "..." is just a special term binding that happens to be
  bound automatically to the argument of the last fact established by
- assume or any local goal.  In contrast to ??thesis, "..." is bound
+ assume or any local goal.  In contrast to ?thesis, "..." is bound
  after the proof is finished.
 *};
 
@@ -112,7 +112,7 @@
   from calculation
     -- {* ... and pick up final result *};
 
-  show ??thesis; .;
+  show ?thesis; .;
 qed;