src/HOL/Predicate_Compile_Examples/Specialisation_Examples.thy
changeset 58249 180f1b3508ed
parent 53374 a14d2a854c02
child 58310 91ea607a34d8
--- a/src/HOL/Predicate_Compile_Examples/Specialisation_Examples.thy	Tue Sep 09 17:51:07 2014 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Specialisation_Examples.thy	Tue Sep 09 20:51:36 2014 +0200
@@ -107,13 +107,13 @@
   "unique [] = True"
 | "unique (x # xs) = (xs\<langle>fst x\<rangle>\<^sub>? = \<bottom> \<and> unique xs)"
 
-datatype type =
+datatype_new type =
     TVar nat
   | Top
   | Fun type type    (infixr "\<rightarrow>" 200)
   | TyAll type type  ("(3\<forall><:_./ _)" [0, 10] 10)
 
-datatype binding = VarB type | TVarB type
+datatype_new binding = VarB type | TVarB type
 type_synonym env = "binding list"
 
 primrec is_TVarB :: "binding \<Rightarrow> bool"
@@ -131,7 +131,7 @@
   "mapB f (VarB T) = VarB (f T)"
 | "mapB f (TVarB T) = TVarB (f T)"
 
-datatype trm =
+datatype_new trm =
     Var nat
   | Abs type trm   ("(3\<lambda>:_./ _)" [0, 10] 10)
   | TAbs type trm  ("(3\<lambda><:_./ _)" [0, 10] 10)