src/Pure/Isar/isar_cmd.ML
changeset 24508 c8b82fec6447
parent 24314 665b3ab2dabe
child 24560 2693220bd77f
equal deleted inserted replaced
24507:ac22a2a67100 24508:c8b82fec6447
   561           (Proof.get_thmss state args)));
   561           (Proof.get_thmss state args)));
   562 
   562 
   563 fun string_of_prop state s =
   563 fun string_of_prop state s =
   564   let
   564   let
   565     val ctxt = Proof.context_of state;
   565     val ctxt = Proof.context_of state;
   566     val prop = ProofContext.read_prop ctxt s;
   566     val prop = Syntax.read_prop ctxt s;
   567   in Pretty.string_of (Pretty.quote (ProofContext.pretty_term ctxt prop)) end;
   567   in Pretty.string_of (Pretty.quote (ProofContext.pretty_term ctxt prop)) end;
   568 
   568 
   569 fun string_of_term state s =
   569 fun string_of_term state s =
   570   let
   570   let
   571     val ctxt = Proof.context_of state;
   571     val ctxt = Proof.context_of state;
   572     val t = ProofContext.read_term ctxt s;
   572     val t = Syntax.read_term ctxt s;
   573     val T = Term.type_of t;
   573     val T = Term.type_of t;
   574   in
   574   in
   575     Pretty.string_of
   575     Pretty.string_of
   576       (Pretty.block [Pretty.quote (ProofContext.pretty_term ctxt t), Pretty.fbrk,
   576       (Pretty.block [Pretty.quote (ProofContext.pretty_term ctxt t), Pretty.fbrk,
   577         Pretty.str "::", Pretty.brk 1, Pretty.quote (ProofContext.pretty_typ ctxt T)])
   577         Pretty.str "::", Pretty.brk 1, Pretty.quote (ProofContext.pretty_typ ctxt T)])