simp only;
authorwenzelm
Tue, 06 Jul 1999 21:11:34 +0200
changeset 6908 1bf0590f4790
parent 6907 870a953e0a8c
child 6909 21601bc4f3c2
simp only;
src/HOL/Isar_examples/Group.thy
--- a/src/HOL/Isar_examples/Group.thy	Tue Jul 06 21:09:23 1999 +0200
+++ b/src/HOL/Isar_examples/Group.thy	Tue Jul 06 21:11:34 1999 +0200
@@ -34,21 +34,21 @@
 theorem group_right_inverse: "x * inv x = (one::'a::group)";
 proof same;
   have "x * inv x = one * (x * inv x)";
-    by (simp add: group_left_unit);
+    by (simp only: group_left_unit);
   also; have "... = (one * x) * inv x";
-    by (simp add: group_assoc);
+    by (simp only: group_assoc);
   also; have "... = inv (inv x) * inv x * x * inv x";
-    by (simp add: group_left_inverse);
+    by (simp only: group_left_inverse);
   also; have "... = inv (inv x) * (inv x * x) * inv x";
-    by (simp add: group_assoc);
+    by (simp only: group_assoc);
   also; have "... = inv (inv x) * one * inv x";
-    by (simp add: group_left_inverse);
+    by (simp only: group_left_inverse);
   also; have "... = inv (inv x) * (one * inv x)";
-    by (simp add: group_assoc);
+    by (simp only: group_assoc);
   also; have "... = inv (inv x) * inv x";
-    by (simp add: group_left_unit);
+    by (simp only: group_left_unit);
   also; have "... = one";
-    by (simp add: group_left_inverse);
+    by (simp only: group_left_inverse);
   finally; show ??thesis; .;
 qed;
 
@@ -60,13 +60,13 @@
 theorem group_right_unit: "x * one = (x::'a::group)";
 proof same;
   have "x * one = x * (inv x * x)";
-    by (simp add: group_left_inverse);
+    by (simp only: group_left_inverse);
   also; have "... = x * inv x * x";
-    by (simp add: group_assoc);
+    by (simp only: group_assoc);
   also; have "... = one * x";
-    by (simp add: group_right_inverse);
+    by (simp only: group_right_inverse);
   also; have "... = x";
-    by (simp add: group_left_unit);
+    by (simp only: group_left_unit);
   finally; show ??thesis; .;
 qed;
 
@@ -87,25 +87,25 @@
 theorem "x * one = (x::'a::group)";
 proof same;
   have "x * one = x * (inv x * x)";
-    by (simp add: group_left_inverse);
+    by (simp only: group_left_inverse);
 
   note calculation = facts
     -- {* first calculational step: init calculation register *};
 
   have "... = x * inv x * x";
-    by (simp add: group_assoc);
+    by (simp only: group_assoc);
 
   note calculation = trans [OF calculation facts]
     -- {* general calculational step: compose with transitivity rule *};
 
   have "... = one * x";
-    by (simp add: group_right_inverse);
+    by (simp only: group_right_inverse);
 
   note calculation = trans [OF calculation facts]
     -- {* general calculational step: compose with transitivity rule *};
 
   have "... = x";
-    by (simp add: group_left_unit);
+    by (simp only: group_left_unit);
 
   note calculation = trans [OF calculation facts]
     -- {* final calculational step: compose with transitivity rule ... *};