diff -r c78b2223f001 -r 6c473ed0ac70 src/HOL/Codegenerator_Test/Code_Test_PolyML.thy --- a/src/HOL/Codegenerator_Test/Code_Test_PolyML.thy Wed Oct 08 00:13:39 2014 +0200 +++ b/src/HOL/Codegenerator_Test/Code_Test_PolyML.thy Wed Oct 08 09:09:12 2014 +0200 @@ -4,7 +4,7 @@ Test case for test_code on PolyML *) -theory Code_Test_PolyML imports Code_Test begin +theory Code_Test_PolyML imports "../Library/Code_Test" begin test_code "14 + 7 * -12 = (140 div -2 :: integer)" in PolyML