Attic/Prove.thy
changeset 1949 0b692f37a771
parent 948 25c4223635f4
child 2171 9697bbf713ec
equal deleted inserted replaced
1948:5abac261b5ce 1949:0b692f37a771
    13     
    13     
    14   fun setup_proof (name_spec, (txt, pos)) lthy =
    14   fun setup_proof (name_spec, (txt, pos)) lthy =
    15   let
    15   let
    16     val trm = ML_Context.evaluate lthy true ("r", r) txt
    16     val trm = ML_Context.evaluate lthy true ("r", r) txt
    17   in
    17   in
    18     Proof.theorem_i NONE (after_qed name_spec) [[(trm,[])]] lthy
    18     Proof.theorem NONE (after_qed name_spec) [[(trm,[])]] lthy
    19   end
    19   end
    20 
    20 
    21   val parser = SpecParse.opt_thm_name ":" -- OuterParse.ML_source
    21   val parser = SpecParse.opt_thm_name ":" -- OuterParse.ML_source
    22 in
    22 in
    23   OuterSyntax.local_theory_to_proof "prove" "proving a proposition" 
    23   OuterSyntax.local_theory_to_proof "prove" "proving a proposition"