src/Pure/Isar/toplevel.ML
changeset 45666 d83797ef0d2d
parent 45488 6d71d9e52369
child 46959 cdc791910460
equal deleted inserted replaced
45665:129db1416717 45666:d83797ef0d2d
   208     NONE => []
   208     NONE => []
   209   | SOME (Theory (gthy, _)) => if prf_only then [] else pretty_context gthy
   209   | SOME (Theory (gthy, _)) => if prf_only then [] else pretty_context gthy
   210   | SOME (Proof (prf, _)) =>
   210   | SOME (Proof (prf, _)) =>
   211       Proof.pretty_state (Proof_Node.position prf) (Proof_Node.current prf)
   211       Proof.pretty_state (Proof_Node.position prf) (Proof_Node.current prf)
   212   | SOME (SkipProof (d, _)) => [Pretty.str ("skipped proof: depth " ^ string_of_int d)])
   212   | SOME (SkipProof (d, _)) => [Pretty.str ("skipped proof: depth " ^ string_of_int d)])
   213   |> Pretty.markup_chunks Markup.state |> Pretty.writeln;
   213   |> Pretty.markup_chunks Isabelle_Markup.state |> Pretty.writeln;
   214 
   214 
   215 fun pretty_abstract state = Pretty.str ("<Isar " ^ str_of_state state ^ ">");
   215 fun pretty_abstract state = Pretty.str ("<Isar " ^ str_of_state state ^ ">");
   216 
   216 
   217 
   217 
   218 
   218