src/Pure/Isar/isar_thy.ML
changeset 7590 76c9e71d491a
parent 7572 6e6dafacbc28
child 7614 88392b7bc549
equal deleted inserted replaced
7589:59663b367833 7590:76c9e71d491a
   340 (* print result *)
   340 (* print result *)
   341 
   341 
   342 local
   342 local
   343 
   343 
   344 fun pretty_result {kind, name, thm} =
   344 fun pretty_result {kind, name, thm} =
   345   Pretty.block [Pretty.str (kind ^ (if name = "" then "" else " " ^ name ^ ":")),
   345   Pretty.block [Pretty.str (kind ^ (if name = "" then "" else " " ^ name) ^ ":"),
   346     Pretty.fbrk, Proof.pretty_thm thm];
   346     Pretty.fbrk, Proof.pretty_thm thm];
   347 
   347 
   348 fun pretty_rule thm =
   348 fun pretty_rule thm =
   349   Pretty.block [Pretty.str "trying to solve goal by rule:", Pretty.fbrk, Proof.pretty_thm thm];
   349   Pretty.block [Pretty.str "trying to solve goal by rule:", Pretty.fbrk, Proof.pretty_thm thm];
   350 
   350