| author | wenzelm | 
| Tue, 08 May 2018 15:41:52 +0200 | |
| changeset 68115 | 23c6ae3dd3a0 | 
| parent 67215 | 03d0c958d65a | 
| child 68189 | 6163c90694ef | 
| permissions | -rw-r--r-- | 
(* Title: Pure/Thy/Sessions.thy Author: Makarius PIDE markup for session ROOT. *) theory Sessions imports Pure keywords "session" :: thy_decl and "description" "options" "sessions" "theories" "document_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