src/HOL/Data_Structures/Tree23_of_List.thy
changeset 79969 4aeb25ba90f3
parent 79490 b287510a4202
--- a/src/HOL/Data_Structures/Tree23_of_List.thy	Sun Mar 24 14:15:10 2024 +0100
+++ b/src/HOL/Data_Structures/Tree23_of_List.thy	Sun Mar 24 14:50:47 2024 +0100
@@ -118,10 +118,10 @@
 
 subsection "Linear running time"
 
-define_time_fun join_adj
-define_time_fun join_all
-define_time_fun leaves
-define_time_fun tree23_of_list
+time_fun join_adj
+time_fun join_all
+time_fun leaves
+time_fun tree23_of_list
 
 lemma T_join_adj: "not_T ts \<Longrightarrow> T_join_adj ts \<le> len ts div 2"
 by(induction ts rule: T_join_adj.induct) auto