src/HOL/Isar_examples/Group.thy
changeset 7133 64c9f2364dae
parent 7005 cc778d613217
child 7356 1714c91b8729
--- a/src/HOL/Isar_examples/Group.thy	Fri Jul 30 13:43:26 1999 +0200
+++ b/src/HOL/Isar_examples/Group.thy	Fri Jul 30 13:44:29 1999 +0200
@@ -32,7 +32,7 @@
 *};
 
 theorem group_right_inverse: "x * inv x = (one::'a::group)";
-proof same;
+proof -;
   have "x * inv x = one * (x * inv x)";
     by (simp only: group_left_unit);
   also; have "... = (one * x) * inv x";
@@ -58,7 +58,7 @@
 *};
 
 theorem group_right_unit: "x * one = (x::'a::group)";
-proof same;
+proof -;
   have "x * one = x * (inv x * x)";
     by (simp only: group_left_inverse);
   also; have "... = x * inv x * x";
@@ -85,7 +85,7 @@
 *};
 
 theorem "x * one = (x::'a::group)";
-proof same;
+proof -;
   have "x * one = x * (inv x * x)";
     by (simp only: group_left_inverse);