src/HOL/Isar_examples/Group.thy
changeset 6881 91a2c8b8269a
parent 6793 88aba7f486cb
child 6892 4a905b4a39c8
--- a/src/HOL/Isar_examples/Group.thy	Thu Jul 01 21:28:49 1999 +0200
+++ b/src/HOL/Isar_examples/Group.thy	Thu Jul 01 21:29:53 1999 +0200
@@ -95,19 +95,19 @@
   have "... = x * inv x * x";
     by (simp add: group_assoc);
 
-  note calculation = trans[APP calculation facts]
+  note calculation = trans[OF calculation facts]
     -- {* general calculational step: compose with transitivity rule *};
 
   have "... = one * x";
     by (simp add: group_right_inverse);
 
-  note calculation = trans[APP calculation facts]
+  note calculation = trans[OF calculation facts]
     -- {* general calculational step: compose with transitivity rule *};
 
   have "... = x";
     by (simp add: group_left_unit);
 
-  note calculation = trans[APP calculation facts]
+  note calculation = trans[OF calculation facts]
     -- {* final calculational step: compose with transitivity rule ... *};
   from calculation
     -- {* ... and pick up final result *};