src/Pure/Pure.thy
changeset 51224 c3e99efacb67
parent 50603 3e3c2af5e8a5
child 51270 17d30843fc3b
equal deleted inserted replaced
51223:c6a8a05ff0a0 51224:c3e99efacb67
    39     "typed_print_translation" "print_ast_translation" "oracle" :: thy_decl % "ML"
    39     "typed_print_translation" "print_ast_translation" "oracle" :: thy_decl % "ML"
    40   and "bundle" :: thy_decl
    40   and "bundle" :: thy_decl
    41   and "include" "including" :: prf_decl
    41   and "include" "including" :: prf_decl
    42   and "print_bundles" :: diag
    42   and "print_bundles" :: diag
    43   and "context" "locale" :: thy_decl
    43   and "context" "locale" :: thy_decl
    44   and "sublocale" "interpretation" :: thy_schematic_goal
    44   and "sublocale" "interpretation" :: thy_goal
    45   and "interpret" :: prf_goal % "proof"  (* FIXME schematic? *)
    45   and "interpret" :: prf_goal % "proof"
    46   and "class" :: thy_decl
    46   and "class" :: thy_decl
    47   and "subclass" :: thy_goal
    47   and "subclass" :: thy_goal
    48   and "instantiation" :: thy_decl
    48   and "instantiation" :: thy_decl
    49   and "instance" :: thy_goal
    49   and "instance" :: thy_goal
    50   and "overloading" :: thy_decl
    50   and "overloading" :: thy_decl