src/Doc/Tutorial/Datatype/Nested.thy
changeset 58860 fee7cfa69c50
parent 58620 7435b6a3f72e
child 67406 23307fd33906
--- a/src/Doc/Tutorial/Datatype/Nested.thy	Sat Nov 01 11:40:55 2014 +0100
+++ b/src/Doc/Tutorial/Datatype/Nested.thy	Sat Nov 01 14:20:38 2014 +0100
@@ -12,7 +12,7 @@
 where function symbols can be applied to a list of arguments:
 *}
 (*<*)hide_const Var(*>*)
-datatype ('v,'f)"term" = Var 'v | App 'f "('v,'f)term list";
+datatype ('v,'f)"term" = Var 'v | App 'f "('v,'f)term list"
 
 text{*\noindent
 Note that we need to quote @{text term} on the left to avoid confusion with
@@ -66,8 +66,8 @@
 *}
 
 lemma subst_id(*<*)(*referred to from ABexpr*)(*>*): "subst  Var t  = (t ::('v,'f)term)  \<and>
-                  substs Var ts = (ts::('v,'f)term list)";
-apply(induct_tac t and ts rule: subst.induct substs.induct, simp_all);
+                  substs Var ts = (ts::('v,'f)term list)"
+apply(induct_tac t and ts rule: subst.induct substs.induct, simp_all)
 done
 
 text{*\noindent