diff -r a1632a5f5fb3 -r 65c775430caa src/Doc/Datatypes/Datatypes.thy --- a/src/Doc/Datatypes/Datatypes.thy Tue Sep 24 20:52:42 2013 +0200 +++ b/src/Doc/Datatypes/Datatypes.thy Tue Sep 24 20:58:27 2013 +0200 @@ -683,7 +683,7 @@ \label{sssec:free-constructor-theorems} *} (*<*) - consts is_Cons :: 'a + consts nonnull :: 'a (*>*) text {* @@ -771,12 +771,12 @@ @{thm list.collapse(1)[no_vars]} \\ @{thm list.collapse(2)[no_vars]} -\item[@{text "t."}\hthm{disc\_exclude}\rm:] ~ \\ +\item[@{text "t."}\hthm{disc\_exclude} @{text "[dest]"}\rm:] ~ \\ These properties are missing for @{typ "'a list"} because there is only one proper discriminator. Had the datatype been introduced with a second -discriminator called @{const is_Cons}, they would have read thusly: \\[\jot] -@{prop "null list \ \ is_Cons list"} \\ -@{prop "is_Cons list \ \ null list"} +discriminator called @{const nonnull}, they would have read thusly: \\[\jot] +@{prop "null list \ \ nonnull list"} \\ +@{prop "nonnull list \ \ null list"} \item[@{text "t."}\hthm{disc\_exhaust} @{text "[case_names C\<^sub>1 \ C\<^sub>n]"}\rm:] ~ \\ @{thm list.disc_exhaust[no_vars]}