src/Pure/Pure.thy
changeset 70205 3293471cf176
parent 70182 ca9dfa7ee3bd
child 70560 7714971a58b5
equal deleted inserted replaced
70204:230188a56a9e 70205:3293471cf176
   123           in thy' end)));
   123           in thy' end)));
   124 
   124 
   125   val _ =
   125   val _ =
   126     Outer_Syntax.local_theory \<^command_keyword>\<open>generate_file\<close>
   126     Outer_Syntax.local_theory \<^command_keyword>\<open>generate_file\<close>
   127       "generate source file, with antiquotations"
   127       "generate source file, with antiquotations"
   128       (Parse.path_binding -- (\<^keyword>\<open>=\<close> |-- Parse.input Parse.embedded)
   128       (Parse.path_binding -- (\<^keyword>\<open>=\<close> |-- Parse.embedded_input)
   129         >> Generated_Files.generate_file_cmd);
   129         >> Generated_Files.generate_file_cmd);
   130 
   130 
   131 
   131 
   132   val files_in_theory =
   132   val files_in_theory =
   133     (Parse.underscore >> K [] || Scan.repeat1 Parse.path_binding) --
   133     (Parse.underscore >> K [] || Scan.repeat1 Parse.path_binding) --