diff -r f1c29e366c09 -r 4aeb25ba90f3 src/HOL/Data_Structures/Define_Time_Function.thy --- a/src/HOL/Data_Structures/Define_Time_Function.thy Sun Mar 24 14:15:10 2024 +0100 +++ b/src/HOL/Data_Structures/Define_Time_Function.thy Sun Mar 24 14:50:47 2024 +0100 @@ -8,10 +8,11 @@ theory Define_Time_Function imports Main - keywords "define_time_fun" :: thy_decl - and "define_time_function" :: thy_goal + keywords "time_fun" :: thy_decl + and "time_function" :: thy_goal + and "time_definition" :: thy_goal and "equations" - and "define_time_0" :: thy_decl + and "time_fun_0" :: thy_decl begin ML_file Define_Time_0.ML @@ -31,17 +32,17 @@ The constant-time assumption for \(=)\ is justified for recursive data types such as lists and trees as long as the comparison is of the form \t = c\ where \c\ is a constant term, for example \xs = []\.\ -define_time_0 "(+)" -define_time_0 "(-)" -define_time_0 "(*)" -define_time_0 "(/)" -define_time_0 "(div)" -define_time_0 "(<)" -define_time_0 "(\)" -define_time_0 "Not" -define_time_0 "(\)" -define_time_0 "(\)" -define_time_0 "Num.numeral_class.numeral" -define_time_0 "(=)" +time_fun_0 "(+)" +time_fun_0 "(-)" +time_fun_0 "(*)" +time_fun_0 "(/)" +time_fun_0 "(div)" +time_fun_0 "(<)" +time_fun_0 "(\)" +time_fun_0 "Not" +time_fun_0 "(\)" +time_fun_0 "(\)" +time_fun_0 "Num.numeral_class.numeral" +time_fun_0 "(=)" end \ No newline at end of file