src/Pure/Pure.thy
changeset 61338 de610e8df459
parent 61337 4645502c3c64
child 61566 c3d6e570ccef
equal deleted inserted replaced
61337:4645502c3c64 61338:de610e8df459
    41   and "subclass" :: thy_goal
    41   and "subclass" :: thy_goal
    42   and "instantiation" :: thy_decl_block
    42   and "instantiation" :: thy_decl_block
    43   and "instance" :: thy_goal
    43   and "instance" :: thy_goal
    44   and "overloading" :: thy_decl_block
    44   and "overloading" :: thy_decl_block
    45   and "code_datatype" :: thy_decl
    45   and "code_datatype" :: thy_decl
    46   and "theorem" "lemma" "corollary" :: thy_goal
    46   and "theorem" "lemma" "corollary" "proposition" :: thy_goal
    47   and "schematic_goal" :: thy_goal
    47   and "schematic_goal" :: thy_goal
    48   and "notepad" :: thy_decl_block
    48   and "notepad" :: thy_decl_block
    49   and "have" :: prf_goal % "proof"
    49   and "have" :: prf_goal % "proof"
    50   and "hence" :: prf_goal % "proof" == "then have"
    50   and "hence" :: prf_goal % "proof" == "then have"
    51   and "show" :: prf_asm_goal % "proof"
    51   and "show" :: prf_asm_goal % "proof"