doc-src/TutorialI/Misc/simp.thy
changeset 12332 aea72a834c85
parent 11494 23a118849801
child 12473 f41e477576b9
--- a/doc-src/TutorialI/Misc/simp.thy	Thu Nov 29 20:02:23 2001 +0100
+++ b/doc-src/TutorialI/Misc/simp.thy	Thu Nov 29 21:12:37 2001 +0100
@@ -42,6 +42,13 @@
   to include simplification rules that can lead to nontermination, either on
   their own or in combination with other simplification rules.
 \end{warn}
+\begin{warn}
+  It is inadvisable to toggle the simplification attribute of a
+  theorem from a parent theory $A$ in a child theory $B$ for good.
+  The reason is that if some theory $C$ is based both on $B$ and (via a
+  differnt path) on $A$, it is not defined what the simplification attribute
+  of that theorem will be in $C$: it could be either.
+\end{warn}
 *} 
 
 subsection{*The {\tt\slshape simp}  Method*}