ProgTutorial/FirstSteps.thy
changeset 400 7675427e311f
parent 394 0019ebf76e10
child 401 36d61044f9bf
--- a/ProgTutorial/FirstSteps.thy	Sat Nov 21 00:29:43 2009 +0100
+++ b/ProgTutorial/FirstSteps.thy	Sun Nov 22 03:13:29 2009 +0100
@@ -838,7 +838,7 @@
   theorem lists; see Section \ref{sec:storing}).
 
   It is also possible to prove lemmas with the antiquotation @{text "@{lemma \<dots> by \<dots>}"}
-  whose first argument is a statement (possibly many of them separated by @{text "and"},
+  whose first argument is a statement (possibly many of them separated by @{text "and"})
   and the second is a proof. For example
 *}