diff -r 4e738f2a97a8 -r e6ae63d1b480 src/HOL/Data_Structures/Tree23_of_List.thy --- a/src/HOL/Data_Structures/Tree23_of_List.thy Tue Dec 05 22:04:01 2023 +0100 +++ b/src/HOL/Data_Structures/Tree23_of_List.thy Wed Dec 06 12:06:29 2023 +0100 @@ -130,7 +130,7 @@ "T_leaves (a # as) = T_leaves as + 1" definition T_tree23_of_list :: "'a list \ nat" where -"T_tree23_of_list as = T_leaves as + T_join_all(leaves as) + 1" +"T_tree23_of_list as = T_leaves as + T_join_all(leaves as)" lemma T_join_adj: "not_T ts \ T_join_adj ts \ len ts div 2" by(induction ts rule: T_join_adj.induct) auto @@ -162,7 +162,7 @@ lemma len_leaves: "len(leaves as) = length as + 1" by(induction as) auto -lemma T_tree23_of_list: "T_tree23_of_list as \ 3*(length as) + 4" +lemma T_tree23_of_list: "T_tree23_of_list as \ 3*(length as) + 3" using T_join_all[of "leaves as"] by(simp add: T_tree23_of_list_def T_leaves len_leaves) end