HOL typedef with explicit dependency checks according to Ondrey Kuncar, 07-Jul-2015, 16-Jul-2015, 30-Jul-2015;
defs.ML: track dependencies also for type constructors;
typedef.ML: add type defined by typedef to dependencies, Abs and Rep now depend on the type;
Pure types and typedecls are final -- no dependencies;
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