src/HOL/Tools/specification_package.ML
changeset 21359 072e83a0b5bb
parent 21116 be58cded79da
child 21434 944f80576be0
equal deleted inserted replaced
21358:f48800c3d573 21359:072e83a0b5bb
   226       fun after_qed [[thm]] = ProofContext.theory (fn thy =>
   226       fun after_qed [[thm]] = ProofContext.theory (fn thy =>
   227         #1 (post_process (add_specification axiomatic (zip3 names cnames overloaded) (thy, thm))));
   227         #1 (post_process (add_specification axiomatic (zip3 names cnames overloaded) (thy, thm))));
   228     in
   228     in
   229       thy
   229       thy
   230       |> ProofContext.init
   230       |> ProofContext.init
   231       |> Proof.theorem_i PureThy.internalK NONE after_qed
   231       |> Proof.theorem_i PureThy.internalK NONE after_qed [[(HOLogic.mk_Trueprop ex_prop, [])]]
   232         (SOME "") ("", []) [(("", []), [(HOLogic.mk_Trueprop ex_prop, [])])]
       
   233     end;
   232     end;
   234 
   233 
   235 
   234 
   236 (* outer syntax *)
   235 (* outer syntax *)
   237 
   236