doc-src/TutorialI/Misc/case_splits.thy
changeset 9723 a977245dfc8a
parent 9721 7e51c9f3d5a0
child 9792 bbefb6ce5cb2
--- a/doc-src/TutorialI/Misc/case_splits.thy	Tue Aug 29 15:43:29 2000 +0200
+++ b/doc-src/TutorialI/Misc/case_splits.thy	Tue Aug 29 16:05:13 2000 +0200
@@ -11,9 +11,9 @@
 
 txt{*\noindent
 can be split into
-\begin{isabellepar}%
+\begin{isabelle}
 ~1.~{\isasymforall}xs.~(xs~=~[]~{\isasymlongrightarrow}~rev~xs~=~[])~{\isasymand}~(xs~{\isasymnoteq}~[]~{\isasymlongrightarrow}~rev~xs~{\isasymnoteq}~[])%
-\end{isabellepar}%
+\end{isabelle}
 by a degenerate form of simplification
 *}
 
@@ -34,10 +34,10 @@
 lemma "(case xs of [] \\<Rightarrow> zs | y#ys \\<Rightarrow> y#(ys@zs)) = xs@zs";
 txt{*\noindent
 becomes
-\begin{isabellepar}%
+\begin{isabelle}
 ~1.~(xs~=~[]~{\isasymlongrightarrow}~zs~=~xs~@~zs)~{\isasymand}\isanewline
 ~~~~({\isasymforall}a~list.~xs~=~a~\#~list~{\isasymlongrightarrow}~a~\#~list~@~zs~=~xs~@~zs)%
-\end{isabellepar}%
+\end{isabelle}
 by typing
 *}