src/HOL/MicroJava/MicroJava.thy
changeset 27680 5a557a5afc48
child 39918 7a1d8b9d17e7
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/MicroJava/MicroJava.thy	Fri Jul 25 12:03:31 2008 +0200
@@ -0,0 +1,15 @@
+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
\ No newline at end of file