src/HOL/MicroJava/BV/BVExample.thy
changeset 17145 e623e57b0f44
parent 16643 39cb9fe20fe3
child 17465 93fc1211603f
--- a/src/HOL/MicroJava/BV/BVExample.thy	Thu Aug 25 16:10:16 2005 +0200
+++ b/src/HOL/MicroJava/BV/BVExample.thy	Thu Aug 25 16:13:09 2005 +0200
@@ -475,12 +475,13 @@
 
 lemmas [code ind] = rtrancl_refl converse_rtrancl_into_rtrancl
 
-generate_code
+code_module BV
+contains
   test1 = "test_kil E list_name [Class list_name] (PrimT Void) 3 0
     [(Suc 0, 2, 8, Xcpt NullPointer)] append_ins"
   test2 = "test_kil E test_name [] (PrimT Void) 3 2 [] make_list_ins"
 
-ML test1
-ML test2
+ML BV.test1
+ML BV.test2
 
 end