diff -r 6e34025981be -r 7c2724cefcb8 src/HOL/Data_Structures/Leftist_Heap.thy --- 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