diff -r d5ddd022a451 -r 47f7263870a0 src/HOL/Data_Structures/Tree234_Set.thy --- a/src/HOL/Data_Structures/Tree234_Set.thy Thu Nov 19 22:35:10 2015 +0100 +++ b/src/HOL/Data_Structures/Tree234_Set.thy Fri Nov 20 12:22:41 2015 +0100 @@ -36,7 +36,7 @@ fun tree\<^sub>i :: "'a up\<^sub>i \ 'a tree234" where "tree\<^sub>i (T\<^sub>i t) = t" | -"tree\<^sub>i (Up\<^sub>i l p r) = Node2 l p r" +"tree\<^sub>i (Up\<^sub>i l a r) = Node2 l a r" fun ins :: "'a::cmp \ 'a tree234 \ 'a up\<^sub>i" where "ins x Leaf = Up\<^sub>i Leaf x Leaf" | @@ -97,8 +97,8 @@ datatype 'a up\<^sub>d = T\<^sub>d "'a tree234" | Up\<^sub>d "'a tree234" fun tree\<^sub>d :: "'a up\<^sub>d \ 'a tree234" where -"tree\<^sub>d (T\<^sub>d x) = x" | -"tree\<^sub>d (Up\<^sub>d x) = x" +"tree\<^sub>d (T\<^sub>d t) = t" | +"tree\<^sub>d (Up\<^sub>d t) = t" fun node21 :: "'a up\<^sub>d \ 'a \ 'a tree234 \ 'a up\<^sub>d" where "node21 (T\<^sub>d l) a r = T\<^sub>d(Node2 l a r)" |