src/Pure/Pure.thy
changeset 73787 493b1ae188da
parent 73312 736b8853189a
child 74171 a9e79c3645c4
equal deleted inserted replaced
73786:18d80cd51823 73787:493b1ae188da
   294   Outer_Syntax.local_theory \<^command_keyword>\<open>local_setup\<close> "ML setup for local theory"
   294   Outer_Syntax.local_theory \<^command_keyword>\<open>local_setup\<close> "ML setup for local theory"
   295     (Parse.ML_source >> Isar_Cmd.local_setup);
   295     (Parse.ML_source >> Isar_Cmd.local_setup);
   296 
   296 
   297 val _ =
   297 val _ =
   298   Outer_Syntax.command \<^command_keyword>\<open>oracle\<close> "declare oracle"
   298   Outer_Syntax.command \<^command_keyword>\<open>oracle\<close> "declare oracle"
   299     (Parse.range Parse.name -- (\<^keyword>\<open>=\<close> |-- Parse.ML_source) >>
   299     (Parse.range Parse.name -- Parse.!!! (\<^keyword>\<open>=\<close> |-- Parse.ML_source) >>
   300       (fn (x, y) => Toplevel.theory (Isar_Cmd.oracle x y)));
   300       (fn (x, y) => Toplevel.theory (Isar_Cmd.oracle x y)));
   301 
   301 
   302 val _ =
   302 val _ =
   303   Outer_Syntax.local_theory \<^command_keyword>\<open>attribute_setup\<close> "define attribute in ML"
   303   Outer_Syntax.local_theory \<^command_keyword>\<open>attribute_setup\<close> "define attribute in ML"
   304     (Parse.name_position --
   304     (Parse.name_position --