doc-src/TutorialI/Misc/simp.thy
changeset 16871 0f483b2632cd
parent 16560 bed540afd4b3
child 19792 e8e3da6d3ff7
equal deleted inserted replaced
16870:a1155e140597 16871:0f483b2632cd
   447 
   447 
   448 \begin{warn}
   448 \begin{warn}
   449 Always use ``\texttt{\_}'' rather than variable names: searching for
   449 Always use ``\texttt{\_}'' rather than variable names: searching for
   450 \texttt{"x + y"} will usually not find any matching theorems
   450 \texttt{"x + y"} will usually not find any matching theorems
   451 because they would need to contain \texttt{x} and~\texttt{y} literally.
   451 because they would need to contain \texttt{x} and~\texttt{y} literally.
   452 
       
   453 When searching for infix operators, do not just type in the symbol,
   452 When searching for infix operators, do not just type in the symbol,
   454 such as~\texttt{+}, but a proper term such as \texttt{"_ + _"}.
   453 such as~\texttt{+}, but a proper term such as \texttt{"_ + _"}.
   455 This remark applies to more complicated syntaxes, too.
   454 This remark applies to more complicated syntaxes, too.
   456 \end{warn}
   455 \end{warn}
   457 
   456