doc-src/TutorialI/Misc/simp.thy
changeset 16871 0f483b2632cd
parent 16560 bed540afd4b3
child 19792 e8e3da6d3ff7
--- a/doc-src/TutorialI/Misc/simp.thy	Mon Jul 18 15:49:34 2005 +0200
+++ b/doc-src/TutorialI/Misc/simp.thy	Tue Jul 19 11:38:45 2005 +0200
@@ -449,7 +449,6 @@
 Always use ``\texttt{\_}'' rather than variable names: searching for
 \texttt{"x + y"} will usually not find any matching theorems
 because they would need to contain \texttt{x} and~\texttt{y} literally.
-
 When searching for infix operators, do not just type in the symbol,
 such as~\texttt{+}, but a proper term such as \texttt{"_ + _"}.
 This remark applies to more complicated syntaxes, too.