src/Pure/Sessions.thy
changeset 75986 27d98da31985
parent 72600 2fa4f25d9d07
--- a/src/Pure/Sessions.thy	Fri Aug 26 21:25:35 2022 +0200
+++ b/src/Pure/Sessions.thy	Fri Aug 26 21:28:26 2022 +0200
@@ -6,15 +6,18 @@
 
 theory Sessions
   imports Pure
-  keywords "session" :: thy_decl
+  keywords "chapter_definition" "session" :: thy_decl
     and "description" "directories" "options" "sessions" "theories"
       "document_theories" "document_files" "export_files" :: quasi_command
     and "global"
 begin
 
 ML \<open>
+  Outer_Syntax.command \<^command_keyword>\<open>chapter_definition\<close> "PIDE markup for session ROOT"
+    Sessions.chapter_definition_parser;
+
   Outer_Syntax.command \<^command_keyword>\<open>session\<close> "PIDE markup for session ROOT"
-    Sessions.command_parser;
+    Sessions.session_parser;
 \<close>
 
 end