src/Doc/Tutorial/Inductive/Mutual.thy
changeset 58774 d6435f0bf966
parent 53015 a1119cf551e8
child 67406 23307fd33906
--- a/src/Doc/Tutorial/Inductive/Mutual.thy	Thu Oct 23 14:43:51 2014 +0200
+++ b/src/Doc/Tutorial/Inductive/Mutual.thy	Thu Oct 23 16:25:08 2014 +0200
@@ -67,7 +67,7 @@
 
 text{*\noindent Everything works as before, except that
 you write \commdx{inductive} instead of \isacommand{inductive\_set} and
-@{prop"evn n"} instead of @{prop"n : even"}.
+@{prop"evn n"} instead of @{prop"n : Even"}.
 When defining an n-ary relation as a predicate, it is recommended to curry
 the predicate: its type should be \mbox{@{text"\<tau>\<^sub>1 \<Rightarrow> \<dots> \<Rightarrow> \<tau>\<^sub>n \<Rightarrow> bool"}}
 rather than