ProgTutorial/Recipes/CallML.thy
changeset 448 957f69b9b7df
parent 441 520127b708e6
child 459 4532577b61e0
--- a/ProgTutorial/Recipes/CallML.thy	Fri Aug 13 18:52:16 2010 +0800
+++ b/ProgTutorial/Recipes/CallML.thy	Sun Aug 22 22:56:52 2010 +0800
@@ -72,7 +72,7 @@
   @{text 4} is not prime: 
 *}
 
-lemma "\<not> prime(4::nat)"
+lemma "\<not> prime (4::nat)"
   apply(rule factor_non_prime)
   apply eval
   done