doc-src/TutorialI/Rules/Forward.thy
changeset 14403 32d1526d3237
parent 13550 5a176b8dda84
child 16417 9bc16273c2d4
--- a/doc-src/TutorialI/Rules/Forward.thy	Fri Feb 20 01:32:59 2004 +0100
+++ b/doc-src/TutorialI/Rules/Forward.thy	Fri Feb 20 14:22:51 2004 +0100
@@ -58,9 +58,22 @@
 lemmas gcd_mult_0 = gcd_mult_distrib2 [of k 1];
 lemmas gcd_mult_1 = gcd_mult_0 [simplified];
 
+lemmas where1 = gcd_mult_distrib2 [where m=1]
+
+lemmas where2 = gcd_mult_distrib2 [where m=1 and k=1]
+
+lemmas where3 = gcd_mult_distrib2 [where m=1 and k="j+k"]
+
 text {*
+example using ``of'':
 @{thm[display] gcd_mult_distrib2 [of _ 1]}
 
+example using ``where'':
+@{thm[display] gcd_mult_distrib2 [where m=1]}
+
+example using ``where'', ``and'':
+@{thm[display] gcd_mult_distrib2 [where m=1 and k="j+k"]}
+
 @{thm[display] gcd_mult_0}
 \rulename{gcd_mult_0}