| changeset 64771 | 23c56f483775 |
| parent 64540 | f1f4ba6d02c9 |
| child 64887 | 266fb24c80bd |
--- a/src/HOL/Library/Tree.thy Wed Dec 07 08:14:40 2016 +0100 +++ b/src/HOL/Library/Tree.thy Wed Jan 04 14:26:08 2017 +0100 @@ -356,8 +356,6 @@ lemma wbalanced_subtrees: "\<lbrakk> wbalanced t; s \<in> subtrees t \<rbrakk> \<Longrightarrow> wbalanced s" using [[simp_depth_limit=1]] by(induction t arbitrary: s) auto -(* show wbalanced \<Longrightarrow> balanced and use that in Balanced.thy *) - subsection \<open>@{const path_len}\<close>