clarified theory location and imports: avoid surprises due to Pure instead of Main (e.g. simpset operations);
tuned headers;
theory MicroJava
imports
"J/JTypeSafe"
"J/Example"
"J/JListExample"
"JVM/JVMListExample"
"JVM/JVMDefensive"
"BV/LBVJVM"
"BV/BVNoTypeError"
"BV/BVExample"
"Comp/CorrComp"
"Comp/CorrCompTp"
begin
end