src/Pure/Proof/proof_syntax.ML
changeset 33388 d64545e6cba5
parent 31943 5e960a0780a2
child 35122 305b3eb5b9d5
equal deleted inserted replaced
33387:acea2f336721 33388:d64545e6cba5
    17   val proof_of: bool -> thm -> Proofterm.proof
    17   val proof_of: bool -> thm -> Proofterm.proof
    18   val pretty_proof: Proof.context -> Proofterm.proof -> Pretty.T
    18   val pretty_proof: Proof.context -> Proofterm.proof -> Pretty.T
    19   val pretty_proof_of: Proof.context -> bool -> thm -> Pretty.T
    19   val pretty_proof_of: Proof.context -> bool -> thm -> Pretty.T
    20 end;
    20 end;
    21 
    21 
    22 structure ProofSyntax : PROOF_SYNTAX =
    22 structure Proof_Syntax : PROOF_SYNTAX =
    23 struct
    23 struct
    24 
    24 
    25 open Proofterm;
    25 open Proofterm;
    26 
    26 
    27 (**** add special syntax for embedding proof terms ****)
    27 (**** add special syntax for embedding proof terms ****)