src/HOL/Data_Structures/Leftist_Heap.thy
changeset 70450 7c2724cefcb8
parent 70363 6d96ee03b62e
child 70585 eecade21bc6a
--- a/src/HOL/Data_Structures/Leftist_Heap.thy	Tue Jul 30 20:09:25 2019 +0200
+++ b/src/HOL/Data_Structures/Leftist_Heap.thy	Wed Jul 31 09:04:00 2019 +0200
@@ -4,7 +4,7 @@
 
 theory Leftist_Heap
 imports
-  Base_FDS
+  "HOL-Library.Pattern_Aliases"
   Tree2
   Priority_Queue_Specs
   Complex_Main