src/Doc/Datatypes/Datatypes.thy
changeset 58339 f6af48bd7c04
parent 58336 a7add8066122
child 58344 ea3d989219b4
--- a/src/Doc/Datatypes/Datatypes.thy	Mon Sep 15 11:37:55 2014 +0200
+++ b/src/Doc/Datatypes/Datatypes.thy	Mon Sep 15 11:54:47 2014 +0200
@@ -1069,6 +1069,10 @@
 The new function returns @{text 1} instead of @{text 0} for some nonrecursive
 constructors. This departure from the old behavior made it possible to implement
 @{const size} in terms of the parameterized function @{text "t.size_t"}.
+Moreover, the new function considers nested occurrences of a value, in the nested
+recursive case. The old behavior can be obtained by disabling the @{text size}
+plugin (Section~\ref{sec:controlling-plugins}) and instantiating the
+@{text size} type class manually.
 
 \item \emph{The internal constructions are completely different.} Proof texts
 that unfold the definition of constants introduced by \keyw{old_datatype} will