doc-src/TutorialI/Trie/Trie.thy
changeset 10971 6852682eaf16
parent 10795 9e888d60d3e5
child 10978 5eebea8f359f
--- a/doc-src/TutorialI/Trie/Trie.thy	Wed Jan 24 11:59:15 2001 +0100
+++ b/doc-src/TutorialI/Trie/Trie.thy	Wed Jan 24 12:29:10 2001 +0100
@@ -130,7 +130,7 @@
 This proof may look surprisingly straightforward. However, note that this
 comes at a cost: the proof script is unreadable because the intermediate
 proof states are invisible, and we rely on the (possibly brittle) magic of
-@{text auto} (@{text simp_all} will not do---try it) to split the subgoals
+@{text auto} (@{text simp_all} will not do --- try it) to split the subgoals
 of the induction up in such a way that case distinction on @{term bs} makes
 sense and solves the proof. Part~\ref{Isar} shows you how to write readable
 and stable proofs.