support for lazy notes in global/local context and Element.Lazy_Notes: name binding and fact without attributes;
register_proofs is now based on lazy thms, but Thm.consolidate_theory will eventually force this (in parallel);
support for lazy notes for locale activation (still inactive);
(* 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
(*>*)