| changeset 71345 | a956b769903e |
| parent 71304 | 9687209ce8cb |
| child 71399 | a77a3506548d |
--- a/src/HOL/Data_Structures/Array_Braun.thy Mon Dec 23 22:35:54 2019 +0100 +++ b/src/HOL/Data_Structures/Array_Braun.thy Tue Dec 24 21:50:02 2019 +0100 @@ -272,7 +272,7 @@ subsubsection \<open>Size\<close> fun diff :: "'a tree \<Rightarrow> nat \<Rightarrow> nat" where -"diff Leaf 0 = 0" | +"diff Leaf _ = 0" | "diff (Node l x r) n = (if n=0 then 1 else if even n then diff r (n div 2 - 1) else diff l (n div 2))" fun size_fast :: "'a tree \<Rightarrow> nat" where