equal
deleted
inserted
replaced
56 |
56 |
57 |
57 |
58 lemmas gcd_mult_0 = gcd_mult_distrib2 [of k 1]; |
58 lemmas gcd_mult_0 = gcd_mult_distrib2 [of k 1]; |
59 lemmas gcd_mult_1 = gcd_mult_0 [simplified]; |
59 lemmas gcd_mult_1 = gcd_mult_0 [simplified]; |
60 |
60 |
61 text {* |
61 lemmas where1 = gcd_mult_distrib2 [where m=1] |
|
62 |
|
63 lemmas where2 = gcd_mult_distrib2 [where m=1 and k=1] |
|
64 |
|
65 lemmas where3 = gcd_mult_distrib2 [where m=1 and k="j+k"] |
|
66 |
|
67 text {* |
|
68 example using ``of'': |
62 @{thm[display] gcd_mult_distrib2 [of _ 1]} |
69 @{thm[display] gcd_mult_distrib2 [of _ 1]} |
|
70 |
|
71 example using ``where'': |
|
72 @{thm[display] gcd_mult_distrib2 [where m=1]} |
|
73 |
|
74 example using ``where'', ``and'': |
|
75 @{thm[display] gcd_mult_distrib2 [where m=1 and k="j+k"]} |
63 |
76 |
64 @{thm[display] gcd_mult_0} |
77 @{thm[display] gcd_mult_0} |
65 \rulename{gcd_mult_0} |
78 \rulename{gcd_mult_0} |
66 |
79 |
67 @{thm[display] gcd_mult_1} |
80 @{thm[display] gcd_mult_1} |