src/Doc/Implementation/Logic.thy
changeset 80590 505f97165f52
parent 80295 8a9588ffc133
child 82256 f65ac4962b66
equal deleted inserted replaced
80589:7849b6370425 80590:505f97165f52
  1291   @{define_ML_type proof_body} \\
  1291   @{define_ML_type proof_body} \\
  1292   @{define_ML Proofterm.proofs: "int Unsynchronized.ref"} \\
  1292   @{define_ML Proofterm.proofs: "int Unsynchronized.ref"} \\
  1293   @{define_ML Proofterm.reconstruct_proof:
  1293   @{define_ML Proofterm.reconstruct_proof:
  1294   "theory -> term -> proof -> proof"} \\
  1294   "theory -> term -> proof -> proof"} \\
  1295   @{define_ML Proofterm.expand_proof: "theory ->
  1295   @{define_ML Proofterm.expand_proof: "theory ->
  1296   (Proofterm.thm_header -> Thm_Name.T option) -> proof -> proof"} \\
  1296   (Proofterm.thm_header -> Thm_Name.P option) -> proof -> proof"} \\
  1297   @{define_ML Proof_Checker.thm_of_proof: "theory -> proof -> thm"} \\
  1297   @{define_ML Proof_Checker.thm_of_proof: "theory -> proof -> thm"} \\
  1298   @{define_ML Proof_Syntax.read_proof: "theory -> bool -> bool -> string -> proof"} \\
  1298   @{define_ML Proof_Syntax.read_proof: "theory -> bool -> bool -> string -> proof"} \\
  1299   @{define_ML Proof_Syntax.pretty_proof: "Proof.context -> proof -> Pretty.T"} \\
  1299   @{define_ML Proof_Syntax.pretty_proof: "Proof.context -> proof -> Pretty.T"} \\
  1300   \end{mldecls}
  1300   \end{mldecls}
  1301 
  1301