| author | paulson <lp15@cam.ac.uk> |
| Sun, 22 Nov 2020 18:26:45 +0000 | |
| changeset 72686 | 703b601d71b5 |
| parent 72600 | 2fa4f25d9d07 |
| child 75986 | 27d98da31985 |
| permissions | -rw-r--r-- |
(* Title: Pure/Sessions.thy Author: Makarius PIDE markup for session ROOT. *) theory Sessions imports Pure keywords "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>session\<close> "PIDE markup for session ROOT" Sessions.command_parser; \<close> end