support for pretty blocks that are "open" and thus have no impact on formatting, only on markup;
effectively revert 2cb4a2970941 and unify pretty-printing in Scala and ML, following Scala before that change;
build error messages are properly formatted again (amending 320bcbf34849): "no_report" markup does not affect its enclosed line break anymore;
(* Title: HOL/MicroJava/DFA/Abstract_BV.thy
Author: Gerwin Klein
Copyright 2003 TUM
*)
section \<open>Abstract Bytecode Verifier\<close>
(*<*)
theory Abstract_BV
imports Typing_Framework_err Kildall LBVCorrect LBVComplete
begin
end
(*>*)