src/HOL/Data_Structures/Leftist_Heap.thy
changeset 68492 c7e0a7bcacaf
parent 68413 b56ed5010e69
child 68600 bdd6536bd57c
--- a/src/HOL/Data_Structures/Leftist_Heap.thy	Sun Jun 24 22:13:23 2018 +0200
+++ b/src/HOL/Data_Structures/Leftist_Heap.thy	Mon Jun 25 14:45:05 2018 +0200
@@ -6,7 +6,7 @@
 imports
   Base_FDS
   Tree2
-  Priority_Queue
+  Priority_Queue_Specs
   Complex_Main
 begin