diff -r 08cc5ab18c84 -r aaa31cd0caef src/HOL/Data_Structures/Brother12_Map.thy --- a/src/HOL/Data_Structures/Brother12_Map.thy Sun Apr 08 09:46:33 2018 +0200 +++ b/src/HOL/Data_Structures/Brother12_Map.thy Sun Apr 08 11:05:52 2018 +0200 @@ -5,7 +5,7 @@ theory Brother12_Map imports Brother12_Set - Map_by_Ordered + Map_Specs begin fun lookup :: "('a \ 'b) bro \ 'a::linorder \ 'b option" where