src/Pure/Sessions.thy
changeset 68292 7ca0c23179e6
parent 68189 6163c90694ef
child 70668 9cac4dec0da9
--- a/src/Pure/Sessions.thy	Sat May 26 19:39:06 2018 +0200
+++ b/src/Pure/Sessions.thy	Sat May 26 19:40:02 2018 +0200
@@ -7,7 +7,8 @@
 theory Sessions
   imports Pure
   keywords "session" :: thy_decl
-    and "description" "options" "sessions" "theories" "document_files" :: quasi_command
+    and "description" "options" "sessions" "theories"
+      "document_files" "export_files" :: quasi_command
     and "global"
 begin