src/HOL/Quotient_Examples/Quotient_Int.thy
changeset 45605 a89b4bc311a5
parent 41467 8fc17c5e11c0
child 47092 fa3538d6004b
--- a/src/HOL/Quotient_Examples/Quotient_Int.thy	Sun Nov 20 20:59:30 2011 +0100
+++ b/src/HOL/Quotient_Examples/Quotient_Int.thy	Sun Nov 20 21:05:23 2011 +0100
@@ -263,11 +263,12 @@
 qed
 
 lemmas int_distrib =
-  left_distrib [of "z1::int" "z2" "w", standard]
-  right_distrib [of "w::int" "z1" "z2", standard]
-  left_diff_distrib [of "z1::int" "z2" "w", standard]
-  right_diff_distrib [of "w::int" "z1" "z2", standard]
-  minus_add_distrib[of "z1::int" "z2", standard]
+  left_distrib [of z1 z2 w]
+  right_distrib [of w z1 z2]
+  left_diff_distrib [of z1 z2 w]
+  right_diff_distrib [of w z1 z2]
+  minus_add_distrib[of z1 z2]
+  for z1 z2 w :: int
 
 lemma int_induct_raw:
   assumes a: "P (0::nat, 0)"