diff -r 4bad9c465eef -r 7e1b66416b7f src/Pure/Pure.thy --- a/src/Pure/Pure.thy Sat Dec 14 22:26:27 2024 +0100 +++ b/src/Pure/Pure.thy Sat Dec 14 23:48:45 2024 +0100 @@ -408,12 +408,12 @@ Parse.!!! (Scan.repeat1 Parse.name_position)); val _ = - Outer_Syntax.command \<^command_keyword>\syntax_consts\ "declare syntax const dependencies" - (syntax_consts >> (Toplevel.theory o Isar_Cmd.syntax_consts)); + Outer_Syntax.local_theory \<^command_keyword>\syntax_consts\ "declare syntax const dependencies" + (syntax_consts >> Isar_Cmd.syntax_consts); val _ = - Outer_Syntax.command \<^command_keyword>\syntax_types\ "declare syntax const dependencies (type names)" - (syntax_consts >> (Toplevel.theory o Isar_Cmd.syntax_types)); + Outer_Syntax.local_theory \<^command_keyword>\syntax_types\ "declare syntax const dependencies (type names)" + (syntax_consts >> Isar_Cmd.syntax_types); val trans_pat = Scan.optional