src/HOL/Codegenerator_Test/Generate_Efficient_Datastructures.thy
changeset 51599 1559e9266280
parent 51161 6ed12ae3b3e1
child 53361 1cb7d3c0cf31
--- a/src/HOL/Codegenerator_Test/Generate_Efficient_Datastructures.thy	Wed Apr 03 10:15:43 2013 +0200
+++ b/src/HOL/Codegenerator_Test/Generate_Efficient_Datastructures.thy	Wed Apr 03 22:26:04 2013 +0200
@@ -6,7 +6,7 @@
 theory Generate_Efficient_Datastructures
 imports
   Candidates
-  "~~/src/HOL/Library/DAList"
+  "~~/src/HOL/Library/DAList_Multiset"
   "~~/src/HOL/Library/RBT_Mapping"
   "~~/src/HOL/Library/RBT_Set"
 begin