src/HOLCF/pcpodef_package.ML
changeset 21359 072e83a0b5bb
parent 21352 073c79be780c
child 21434 944f80576be0
equal deleted inserted replaced
21358:f48800c3d573 21359:072e83a0b5bb
   171     val (goal, pcpodef_result) =
   171     val (goal, pcpodef_result) =
   172       prepare_pcpodef prep_term pcpo def name typ set opt_morphs thy;
   172       prepare_pcpodef prep_term pcpo def name typ set opt_morphs thy;
   173     fun after_qed [[th]] = ProofContext.theory (pcpodef_result th);
   173     fun after_qed [[th]] = ProofContext.theory (pcpodef_result th);
   174   in
   174   in
   175     ProofContext.init thy
   175     ProofContext.init thy
   176     |> Proof.theorem_i PureThy.internalK NONE after_qed NONE ("", []) [(("", []), [(goal, [])])]
   176     |> Proof.theorem_i PureThy.internalK NONE after_qed [[(goal, [])]]
   177   end;
   177   end;
   178 
   178 
   179 fun pcpodef_proof x = gen_pcpodef_proof ProofContext.read_term true x;
   179 fun pcpodef_proof x = gen_pcpodef_proof ProofContext.read_term true x;
   180 fun pcpodef_proof_i x = gen_pcpodef_proof ProofContext.cert_term true x;
   180 fun pcpodef_proof_i x = gen_pcpodef_proof ProofContext.cert_term true x;
   181 
   181