ProgTutorial/Parsing.thy
changeset 287 4b75f40b3e6c
parent 286 ff0b3d87a551
child 299 d0b81d6e1b28
--- a/ProgTutorial/Parsing.thy	Wed Jul 22 15:14:29 2009 +0200
+++ b/ProgTutorial/Parsing.thy	Wed Jul 22 15:15:22 2009 +0200
@@ -1099,7 +1099,7 @@
   parser @{ML Scan.succeed}) and only applies a single tactic, namely the tactic which 
   applies @{thm [source] conjE} and then @{thm [source] conjI}. The function 
   @{ML [index] SIMPLE_METHOD}
-  turns such a tactic into a method. The method @{text "foobar"} can be used as follows
+  turns such a tactic into a method. The method @{text "foo"} can be used as follows
 *}
 
 lemma shows "A \<and> B \<Longrightarrow> C \<and> D"