src/HOL/Codegenerator_Test/Code_Test_OCaml.thy
changeset 81714 5e3dd01a9eb2
parent 81713 378b9d6c52b2
child 81815 0b31f0909060
--- a/src/HOL/Codegenerator_Test/Code_Test_OCaml.thy	Sat Jan 04 14:41:30 2025 +0100
+++ b/src/HOL/Codegenerator_Test/Code_Test_OCaml.thy	Sat Jan 04 17:38:45 2025 +0100
@@ -1,11 +1,9 @@
 (*  Title:      HOL/Codegenerator_Test/Code_Test_OCaml.thy
     Author:     Andreas Lochbihler, ETH Zurich
-    Author:     Florian Haftmann, TU Muenchen
 *)
 
 theory Code_Test_OCaml
 imports
-  "HOL-Library.Code_Target_Bit_Shifts"
   "HOL-Library.Code_Test"
   Code_Lazy_Test
 begin