| author | wenzelm |
| Tue, 04 Jun 2019 20:49:33 +0200 | |
| changeset 70326 | aa7c49651f4e |
| parent 68292 | 7ca0c23179e6 |
| child 70668 | 9cac4dec0da9 |
| 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" "options" "sessions" "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