equal
deleted
inserted
replaced
1113 % |
1113 % |
1114 \[@{thm at_simps(1)[no_vars]} |
1114 \[@{thm at_simps(1)[no_vars]} |
1115 \qquad @{thm at_simps(2)[no_vars]}\] |
1115 \qquad @{thm at_simps(2)[no_vars]}\] |
1116 % |
1116 % |
1117 The next example is defined using \keyw{fun} to escape the syntactic |
1117 The next example is defined using \keyw{fun} to escape the syntactic |
1118 restrictions imposed on primitive recursive functions. The |
1118 restrictions imposed on primitively recursive functions. The |
1119 @{command datatype_new_compat} command is needed to register new-style datatypes |
1119 @{command datatype_new_compat} command is needed to register new-style datatypes |
1120 for use with \keyw{fun} and \keyw{function} |
1120 for use with \keyw{fun} and \keyw{function} |
1121 (Section~\ref{sssec:datatype-new-compat}): |
1121 (Section~\ref{sssec:datatype-new-compat}): |
1122 *} |
1122 *} |
1123 |
1123 |