src/HOL/Library/Tree.thy
changeset 58310 91ea607a34d8
parent 57687 cca7e8788481
child 58424 cbbba613b6ab
--- a/src/HOL/Library/Tree.thy	Thu Sep 11 19:26:59 2014 +0200
+++ b/src/HOL/Library/Tree.thy	Thu Sep 11 19:32:36 2014 +0200
@@ -6,7 +6,7 @@
 imports Main
 begin
 
-datatype_new 'a tree = Leaf | Node (left: "'a tree") (val: 'a) (right: "'a tree")
+datatype 'a tree = Leaf | Node (left: "'a tree") (val: 'a) (right: "'a tree")
   where
     "left Leaf = Leaf"
   | "right Leaf = Leaf"