doc-src/TutorialI/Misc/def_rewr.thy
changeset 9723 a977245dfc8a
parent 9689 751fde5307e4
--- a/doc-src/TutorialI/Misc/def_rewr.thy	Tue Aug 29 15:43:29 2000 +0200
+++ b/doc-src/TutorialI/Misc/def_rewr.thy	Tue Aug 29 16:05:13 2000 +0200
@@ -28,9 +28,9 @@
 
 txt{*\noindent
 In this particular case, the resulting goal
-\begin{isabellepar}%
+\begin{isabelle}
 ~1.~A~{\isasymand}~{\isasymnot}~{\isasymnot}~A~{\isasymor}~{\isasymnot}~A~{\isasymand}~{\isasymnot}~A%
-\end{isabellepar}%
+\end{isabelle}
 can be proved by simplification. Thus we could have proved the lemma outright
 *}(*<*)oops;lemma "exor A (\\<not>A)";(*>*)
 by(simp add: exor_def)