src/Pure/Pure.thy
changeset 63270 7dd3ee7ee422
parent 63180 ddfd021884b4
child 63271 ecaa677d20bc
equal deleted inserted replaced
63269:27d51aa2d711 63270:7dd3ee7ee422
    30   and "setup" "local_setup" "attribute_setup" "method_setup"
    30   and "setup" "local_setup" "attribute_setup" "method_setup"
    31     "declaration" "syntax_declaration"
    31     "declaration" "syntax_declaration"
    32     "parse_ast_translation" "parse_translation" "print_translation"
    32     "parse_ast_translation" "parse_translation" "print_translation"
    33     "typed_print_translation" "print_ast_translation" "oracle" :: thy_decl % "ML"
    33     "typed_print_translation" "print_ast_translation" "oracle" :: thy_decl % "ML"
    34   and "bundle" :: thy_decl
    34   and "bundle" :: thy_decl
       
    35   and "bundle_target" :: thy_decl_block
    35   and "include" "including" :: prf_decl
    36   and "include" "including" :: prf_decl
    36   and "print_bundles" :: diag
    37   and "print_bundles" :: diag
    37   and "context" "locale" "experiment" :: thy_decl_block
    38   and "context" "locale" "experiment" :: thy_decl_block
    38   and "interpret" :: prf_goal % "proof"
    39   and "interpret" :: prf_goal % "proof"
    39   and "interpretation" "global_interpretation" "sublocale" :: thy_goal
    40   and "interpretation" "global_interpretation" "sublocale" :: thy_goal
   494   Outer_Syntax.local_theory @{command_keyword bundle} "define bundle of declarations"
   495   Outer_Syntax.local_theory @{command_keyword bundle} "define bundle of declarations"
   495     ((Parse.binding --| @{keyword "="}) -- Parse.thms1 -- Parse.for_fixes
   496     ((Parse.binding --| @{keyword "="}) -- Parse.thms1 -- Parse.for_fixes
   496       >> (uncurry Bundle.bundle_cmd));
   497       >> (uncurry Bundle.bundle_cmd));
   497 
   498 
   498 val _ =
   499 val _ =
       
   500   Outer_Syntax.command @{command_keyword bundle_target} "define bundle of declarations"
       
   501     (Parse.binding --| Parse.begin >> (Toplevel.begin_local_theory true o Bundle.init));
       
   502 
       
   503 val _ =
   499   Outer_Syntax.command @{command_keyword include}
   504   Outer_Syntax.command @{command_keyword include}
   500     "include declarations from bundle in proof body"
   505     "include declarations from bundle in proof body"
   501     (Scan.repeat1 (Parse.position Parse.name) >> (Toplevel.proof o Bundle.include_cmd));
   506     (Scan.repeat1 (Parse.position Parse.name) >> (Toplevel.proof o Bundle.include_cmd));
   502 
   507 
   503 val _ =
   508 val _ =