src/Pure/Pure.thy
changeset 50128 599c935aac82
parent 49569 7b6aaf446496
child 50603 3e3c2af5e8a5
equal deleted inserted replaced
50127:ff0b52a6d72f 50128:599c935aac82
    50   and "overloading" :: thy_decl
    50   and "overloading" :: thy_decl
    51   and "code_datatype" :: thy_decl
    51   and "code_datatype" :: thy_decl
    52   and "theorem" "lemma" "corollary" :: thy_goal
    52   and "theorem" "lemma" "corollary" :: thy_goal
    53   and "schematic_theorem" "schematic_lemma" "schematic_corollary" :: thy_schematic_goal
    53   and "schematic_theorem" "schematic_lemma" "schematic_corollary" :: thy_schematic_goal
    54   and "notepad" :: thy_decl
    54   and "notepad" :: thy_decl
    55   and "have" "hence" :: prf_goal % "proof"
    55   and "have" :: prf_goal % "proof"
    56   and "show" "thus" :: prf_asm_goal % "proof"
    56   and "hence" :: prf_goal % "proof" == "then have"
       
    57   and "show" :: prf_asm_goal % "proof"
       
    58   and "thus" :: prf_asm_goal % "proof" == "then show"
    57   and "then" "from" "with" :: prf_chain % "proof"
    59   and "then" "from" "with" :: prf_chain % "proof"
    58   and "note" "using" "unfolding" :: prf_decl % "proof"
    60   and "note" "using" "unfolding" :: prf_decl % "proof"
    59   and "fix" "assume" "presume" "def" :: prf_asm % "proof"
    61   and "fix" "assume" "presume" "def" :: prf_asm % "proof"
    60   and "obtain" "guess" :: prf_asm_goal % "proof"
    62   and "obtain" "guess" :: prf_asm_goal % "proof"
    61   and "let" "write" :: prf_decl % "proof"
    63   and "let" "write" :: prf_decl % "proof"
    64   and "}" :: prf_close % "proof"
    66   and "}" :: prf_close % "proof"
    65   and "next" :: prf_block % "proof"
    67   and "next" :: prf_block % "proof"
    66   and "qed" :: qed_block % "proof"
    68   and "qed" :: qed_block % "proof"
    67   and "by" ".." "." "done" "sorry" :: "qed" % "proof"
    69   and "by" ".." "." "done" "sorry" :: "qed" % "proof"
    68   and "oops" :: qed_global % "proof"
    70   and "oops" :: qed_global % "proof"
    69   and "defer" "prefer" "apply" "apply_end" :: prf_script % "proof"
    71   and "defer" "prefer" "apply" :: prf_script % "proof"
       
    72   and "apply_end" :: prf_script % "proof" == ""
    70   and "proof" :: prf_block % "proof"
    73   and "proof" :: prf_block % "proof"
    71   and "also" "moreover" :: prf_decl % "proof"
    74   and "also" "moreover" :: prf_decl % "proof"
    72   and "finally" "ultimately" :: prf_chain % "proof"
    75   and "finally" "ultimately" :: prf_chain % "proof"
    73   and "back" :: prf_script % "proof"
    76   and "back" :: prf_script % "proof"
    74   and "Isabelle.command" :: control
    77   and "Isabelle.command" :: control