src/HOL/Data_Structures/Define_Time_Function.thy
changeset 81088 28ef01901650
parent 80738 6adf6cc82013
child 81147 503e5280ba72
--- a/src/HOL/Data_Structures/Define_Time_Function.thy	Wed Oct 02 13:51:45 2024 +0200
+++ b/src/HOL/Data_Structures/Define_Time_Function.thy	Wed Oct 02 18:32:36 2024 +0200
@@ -10,8 +10,8 @@
 theory Define_Time_Function
   imports Main
   keywords "time_fun" :: thy_decl
-    and    "time_function" :: thy_goal
-    and    "time_definition" :: thy_goal
+    and    "time_function" :: thy_decl
+    and    "time_definition" :: thy_decl
     and    "equations"
     and    "time_fun_0" :: thy_decl
 begin