src/Pure/Isar/isar_cmd.ML
changeset 26626 c6231d64d264
parent 26599 791e4b436f8a
child 26671 c95590e01df5
equal deleted inserted replaced
26625:e0cc4169626e 26626:c6231d64d264
   562 fun string_of_prfs full state arg =
   562 fun string_of_prfs full state arg =
   563   Pretty.string_of (case arg of
   563   Pretty.string_of (case arg of
   564       NONE =>
   564       NONE =>
   565         let
   565         let
   566           val (ctxt, (_, thm)) = Proof.get_goal state;
   566           val (ctxt, (_, thm)) = Proof.get_goal state;
   567           val {thy, der = (_, prf), ...} = Thm.rep_thm thm;
   567           val thy = ProofContext.theory_of ctxt;
       
   568           val prf = Thm.proof_of thm;
   568           val prop = Thm.full_prop_of thm;
   569           val prop = Thm.full_prop_of thm;
   569           val prf' = Proofterm.rewrite_proof_notypes ([], []) prf
   570           val prf' = Proofterm.rewrite_proof_notypes ([], []) prf
   570         in
   571         in
   571           ProofContext.pretty_proof ctxt
   572           ProofContext.pretty_proof ctxt
   572             (if full then Reconstruct.reconstruct_proof thy prop prf' else prf')
   573             (if full then Reconstruct.reconstruct_proof thy prop prf' else prf')