src/HOL/Datatype_Examples/Process.thy
changeset 58310 91ea607a34d8
parent 58309 a09ec6daaa19
child 58607 1f90ea1b4010
--- a/src/HOL/Datatype_Examples/Process.thy	Thu Sep 11 19:26:59 2014 +0200
+++ b/src/HOL/Datatype_Examples/Process.thy	Thu Sep 11 19:32:36 2014 +0200
@@ -79,7 +79,7 @@
 
 subsection{* Multi-guard fixpoint definitions, simulated with auxiliary arguments *}
 
-datatype_new x_y_ax = x | y | ax
+datatype x_y_ax = x | y | ax
 
 primcorec F :: "x_y_ax \<Rightarrow> char list process" where
   "xyax = x \<Longrightarrow> isChoice (F xyax)"
@@ -106,7 +106,7 @@
 hide_const x y ax X Y AX
 
 (* Process terms *)
-datatype_new ('a,'pvar) process_term =
+datatype ('a,'pvar) process_term =
  VAR 'pvar |
  PROC "'a process" |
  ACT 'a "('a,'pvar) process_term" | CH "('a,'pvar) process_term" "('a,'pvar) process_term"