src/HOL/Data_Structures/Tree23.thy
changeset 72566 831f17da1aab
parent 70273 acc1749c2be9
child 72586 e3ba2578ad9d
equal deleted inserted replaced
72565:ed5b907bbf50 72566:831f17da1aab
    30 
    30 
    31 instance ..
    31 instance ..
    32 
    32 
    33 end
    33 end
    34 
    34 
    35 text \<open>Balanced:\<close>
    35 text \<open>Completeness:\<close>
    36 
    36 
    37 fun complete :: "'a tree23 \<Rightarrow> bool" where
    37 fun complete :: "'a tree23 \<Rightarrow> bool" where
    38 "complete Leaf = True" |
    38 "complete Leaf = True" |
    39 "complete (Node2 l _ r) = (complete l & complete r & height l = height r)" |
    39 "complete (Node2 l _ r) = (complete l & complete r & height l = height r)" |
    40 "complete (Node3 l _ m _ r) =
    40 "complete (Node3 l _ m _ r) =