changeset 58249 | 180f1b3508ed |
parent 52666 | 391913d17d15 |
child 58310 | 91ea607a34d8 |
--- a/src/HOL/Predicate_Compile_Examples/Lambda_Example.thy Tue Sep 09 17:51:07 2014 +0200 +++ b/src/HOL/Predicate_Compile_Examples/Lambda_Example.thy Tue Sep 09 20:51:36 2014 +0200 @@ -4,11 +4,11 @@ subsection {* Lambda *} -datatype type = +datatype_new type = Atom nat | Fun type type (infixr "\<Rightarrow>" 200) -datatype dB = +datatype_new dB = Var nat | App dB dB (infixl "\<degree>" 200) | Abs type dB