src/HOL/Data_Structures/Lookup2.thy
changeset 68413 b56ed5010e69
parent 67965 aaa31cd0caef
child 70755 3fb16bed5d6c
--- a/src/HOL/Data_Structures/Lookup2.thy	Mon Jun 11 08:15:43 2018 +0200
+++ b/src/HOL/Data_Structures/Lookup2.thy	Mon Jun 11 16:29:27 2018 +0200
@@ -11,7 +11,7 @@
 
 fun lookup :: "('a::linorder * 'b, 'c) tree \<Rightarrow> 'a \<Rightarrow> 'b option" where
 "lookup Leaf x = None" |
-"lookup (Node _ l (a,b) r) x =
+"lookup (Node l (a,b) _ r) x =
   (case cmp x a of LT \<Rightarrow> lookup l x | GT \<Rightarrow> lookup r x | EQ \<Rightarrow> Some b)"
 
 lemma lookup_map_of: