changeset 67965 | aaa31cd0caef |
parent 67406 | 23307fd33906 |
child 68020 | 6aade817bee5 |
--- 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 \<times> 'b) bro \<Rightarrow> 'a::linorder \<Rightarrow> 'b option" where