ProgTutorial/FirstSteps.thy
changeset 269 3e084d62885c
parent 268 509e2ca547db
child 271 949957531f63
--- a/ProgTutorial/FirstSteps.thy	Tue Jul 21 11:59:09 2009 +0200
+++ b/ProgTutorial/FirstSteps.thy	Tue Jul 21 12:05:15 2009 +0200
@@ -803,7 +803,7 @@
   | is_all _ = false*}
 
 text {* 
-  will not correctly match the formula @{prop "\<forall>x::nat. P x"}: 
+  will not correctly match the formula @{prop[source] "\<forall>x::nat. P x"}: 
 
   @{ML_response [display,gray] "is_all @{term \"\<forall>x::nat. P x\"}" "false"}