Prove.thy
author Cezary Kaliszyk <kaliszyk@in.tum.de>
Tue, 22 Sep 2009 17:39:52 +0200
changeset 29 2b59bf690633
parent 6 6a1b4c22a386
child 46 e801b929216b
permissions -rw-r--r--
Proper definition of CARD and some properties of it. Translation should now support Pure assumptions and Trueprops anywhere, but a problem needs to be fixed with the tactic.

theory Prove
imports Main
begin

ML {*
val r = ref (NONE:(unit -> term) option)
*}
ML {*
let
   fun setup_proof (txt, pos) lthy =
   let
     val trm = ML_Context.evaluate lthy true ("r", r) txt
   in
       Proof.theorem_i NONE (K I) [[(trm,[])]] lthy
   end;

   val setup_proof_parser = OuterParse.ML_source >> setup_proof
        
   val kind = OuterKeyword.thy_goal
in
   OuterSyntax.local_theory_to_proof "prove" "proving a proposition" 
    kind setup_proof_parser
end
*}

end