src/HOL/Tools/specification_package.ML
changeset 21434 944f80576be0
parent 21359 072e83a0b5bb
child 21858 05f57309170c
equal deleted inserted replaced
21433:89104dca628e 21434:944f80576be0
   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 [[(HOLogic.mk_Trueprop ex_prop, [])]]
   231       |> Proof.theorem_i NONE after_qed [[(HOLogic.mk_Trueprop ex_prop, [])]]
   232     end;
   232     end;
   233 
   233 
   234 
   234 
   235 (* outer syntax *)
   235 (* outer syntax *)
   236 
   236