src/Doc/Tutorial/Misc/case_exprs.thy
changeset 58860 fee7cfa69c50
parent 48985 5386df44a037
child 67406 23307fd33906
--- a/src/Doc/Tutorial/Misc/case_exprs.thy	Sat Nov 01 11:40:55 2014 +0100
+++ b/src/Doc/Tutorial/Misc/case_exprs.thy	Sat Nov 01 14:20:38 2014 +0100
@@ -52,8 +52,8 @@
 by \methdx{case_tac}.  Here is a trivial example:
 *}
 
-lemma "(case xs of [] \<Rightarrow> [] | y#ys \<Rightarrow> xs) = xs";
-apply(case_tac xs);
+lemma "(case xs of [] \<Rightarrow> [] | y#ys \<Rightarrow> xs) = xs"
+apply(case_tac xs)
 
 txt{*\noindent
 results in the proof state