author | nipkow |
Wed, 18 Jan 2017 21:03:39 +0100 | |
changeset 64921 | 1cbfe46ad6b1 |
parent 64920 | 31044168af84 |
child 64922 | 3fb4d7d00230 |
--- a/src/HOL/Library/Tree.thy Wed Jan 18 17:56:52 2017 +0100 +++ b/src/HOL/Library/Tree.thy Wed Jan 18 21:03:39 2017 +0100 @@ -357,7 +357,7 @@ text \<open>The internal path length of a tree:\<close> lemma ipl_if_complete: "complete t - \<Longrightarrow> ipl t = (let n = height t in 2 + n*2^n - 2^(n+1))" + \<Longrightarrow> ipl t = (let h = height t in 2 + h*2^h - 2^(h+1))" proof(induction t) case (Node l x r) have *: "2^(n+1) \<le> 2 + n*2^n" for n :: nat