src/Pure/Proof/proof_syntax.ML
changeset 70839 2136e4670ad2
parent 70813 83b7d1927fda
child 70914 05c4c6a99b3f
equal deleted inserted replaced
70838:e381e2624077 70839:2136e4670ad2
    11   val read_term: theory -> bool -> typ -> string -> term
    11   val read_term: theory -> bool -> typ -> string -> term
    12   val read_proof: theory -> bool -> bool -> string -> Proofterm.proof
    12   val read_proof: theory -> bool -> bool -> string -> Proofterm.proof
    13   val proof_syntax: Proofterm.proof -> theory -> theory
    13   val proof_syntax: Proofterm.proof -> theory -> theory
    14   val proof_of: bool -> thm -> Proofterm.proof
    14   val proof_of: bool -> thm -> Proofterm.proof
    15   val pretty_proof: Proof.context -> Proofterm.proof -> Pretty.T
    15   val pretty_proof: Proof.context -> Proofterm.proof -> Pretty.T
    16   val pretty_clean_proof_of: Proof.context -> bool -> thm -> Pretty.T
    16   val pretty_standard_proof_of: Proof.context -> bool -> thm -> Pretty.T
    17 end;
    17 end;
    18 
    18 
    19 structure Proof_Syntax : PROOF_SYNTAX =
    19 structure Proof_Syntax : PROOF_SYNTAX =
    20 struct
    20 struct
    21 
    21 
   193 fun pretty_proof ctxt prf =
   193 fun pretty_proof ctxt prf =
   194   Proof_Context.pretty_term_abbrev
   194   Proof_Context.pretty_term_abbrev
   195     (Proof_Context.transfer (proof_syntax prf (Proof_Context.theory_of ctxt)) ctxt)
   195     (Proof_Context.transfer (proof_syntax prf (Proof_Context.theory_of ctxt)) ctxt)
   196     (Proofterm.term_of_proof prf);
   196     (Proofterm.term_of_proof prf);
   197 
   197 
   198 fun pretty_clean_proof_of ctxt full thm =
   198 fun pretty_standard_proof_of ctxt full thm =
   199   pretty_proof ctxt (Thm.clean_proof_of full thm);
   199   pretty_proof ctxt (Thm.standard_proof_of full thm);
   200 
   200 
   201 end;
   201 end;