changeset 58249 | 180f1b3508ed |
parent 47836 | 471cc845430b |
child 58310 | 91ea607a34d8 |
--- a/src/HOL/ex/Termination.thy Tue Sep 09 17:51:07 2014 +0200 +++ b/src/HOL/ex/Termination.thy Tue Sep 09 20:51:36 2014 +0200 @@ -118,7 +118,7 @@ subsection {* Simple examples with other datatypes than nat, e.g. trees and lists *} -datatype tree = Node | Branch tree tree +datatype_new tree = Node | Branch tree tree fun g_tree :: "tree * tree \<Rightarrow> tree" where