src/Doc/Codegen/Introduction.thy
changeset 58305 57752a91eec4
parent 48985 5386df44a037
child 58310 91ea607a34d8
--- a/src/Doc/Codegen/Introduction.thy	Thu Sep 11 18:54:36 2014 +0200
+++ b/src/Doc/Codegen/Introduction.thy	Thu Sep 11 18:54:36 2014 +0200
@@ -35,7 +35,7 @@
 subsection {* A quick start with the Isabelle/HOL toolbox \label{sec:queue_example} *}
 
 text {*
-  In a HOL theory, the @{command_def datatype} and @{command_def
+  In a HOL theory, the @{command_def datatype_new} and @{command_def
   definition}/@{command_def primrec}/@{command_def fun} declarations
   form the core of a functional programming language.  By default
   equational theorems stemming from those are used for generated code,
@@ -45,7 +45,7 @@
   For example, here a simple \qt{implementation} of amortised queues:
 *}
 
-datatype %quote 'a queue = AQueue "'a list" "'a list"
+datatype_new %quote 'a queue = AQueue "'a list" "'a list"
 
 definition %quote empty :: "'a queue" where
   "empty = AQueue [] []"