src/HOL/Codegenerator_Test/Code_Test_OCaml.thy
changeset 65552 f533820e7248
parent 63167 0909deb8059b
child 66453 cc19f7ca2ed6
--- a/src/HOL/Codegenerator_Test/Code_Test_OCaml.thy	Sat Apr 22 12:52:55 2017 +0200
+++ b/src/HOL/Codegenerator_Test/Code_Test_OCaml.thy	Sat Apr 22 22:01:35 2017 +0200
@@ -4,7 +4,7 @@
 Test case for test_code on OCaml
 *)
 
-theory Code_Test_OCaml imports  "../Library/Code_Test" "../GCD" begin
+theory Code_Test_OCaml imports  "../Library/Code_Test" begin
 
 test_code "14 + 7 * -12 = (140 div -2 :: integer)" in OCaml