ProgTutorial/FirstSteps.thy
changeset 275 4b97bff55650
parent 274 f9f3ecc949c5
child 276 682d4711f91e
--- a/ProgTutorial/FirstSteps.thy	Tue Jul 21 13:22:17 2009 +0200
+++ b/ProgTutorial/FirstSteps.thy	Tue Jul 21 13:27:39 2009 +0200
@@ -935,7 +935,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"}