src/Pure/Pure.thy
changeset 70055 36fb663145e5
parent 70054 a884b2967dd7
child 70056 25c0ad612d62
equal deleted inserted replaced
70054:a884b2967dd7 70055:36fb663145e5
   155     Outer_Syntax.command \<^command_keyword>\<open>compile_generated_files\<close>
   155     Outer_Syntax.command \<^command_keyword>\<open>compile_generated_files\<close>
   156       "compile generated files and export results"
   156       "compile generated files and export results"
   157       (Parse.and_list files_in --
   157       (Parse.and_list files_in --
   158         Scan.optional (\<^keyword>\<open>external_files\<close> |-- Parse.!!! (Parse.and_list1 external_files)) [] --
   158         Scan.optional (\<^keyword>\<open>external_files\<close> |-- Parse.!!! (Parse.and_list1 external_files)) [] --
   159         Scan.optional (\<^keyword>\<open>export_files\<close> |-- Parse.!!! (Parse.and_list1 export_files)) [] --
   159         Scan.optional (\<^keyword>\<open>export_files\<close> |-- Parse.!!! (Parse.and_list1 export_files)) [] --
   160         Scan.optional (\<^keyword>\<open>export_prefix\<close> |-- Parse.path_binding) ("compiled", Position.none) --
   160         Scan.optional (\<^keyword>\<open>export_prefix\<close> |-- Parse.path_binding) ("", Position.none) --
   161         (Parse.where_ |-- Parse.!!! Parse.ML_source)
   161         (Parse.where_ |-- Parse.!!! Parse.ML_source)
   162         >> (fn ((((args, external), export), export_prefix), source) =>
   162         >> (fn ((((args, external), export), export_prefix), source) =>
   163           Toplevel.keep (fn st =>
   163           Toplevel.keep (fn st =>
   164             Generated_Files.compile_generated_files_cmd
   164             Generated_Files.compile_generated_files_cmd
   165               (Toplevel.context_of st) args external export export_prefix source)));
   165               (Toplevel.context_of st) args external export export_prefix source)));