proper instantiation of mk_left_commute;
authorwenzelm
Thu, 08 Aug 2002 23:48:31 +0200
changeset 13483 0e6adce08fb0
parent 13482 2bb7200a99cf
child 13484 d8f5d3391766
proper instantiation of mk_left_commute;
src/HOL/Library/Ring_and_Field.thy
--- a/src/HOL/Library/Ring_and_Field.thy	Thu Aug 08 23:47:41 2002 +0200
+++ b/src/HOL/Library/Ring_and_Field.thy	Thu Aug 08 23:48:31 2002 +0200
@@ -90,7 +90,7 @@
 qed
 
 lemma mult_left_commute: "a * (b * c) = b * (a * (c::'a::ring))"
-by(rule mk_left_commute[OF mult_assoc mult_commute])
+  by (rule mk_left_commute [of "op *", OF mult_assoc mult_commute])
 
 theorems ring_mult_ac = mult_assoc mult_commute mult_left_commute