# HG changeset patch # User nipkow # Date 1483536368 -3600 # Node ID 23c56f483775fdcfbb9fe7bf730d1cc137892279 # Parent 3d4331b658613805a57bd86fbdd7de33f6ef296b tuned diff -r 3d4331b65861 -r 23c56f483775 src/HOL/Library/Tree.thy --- 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: "\ wbalanced t; s \ subtrees t \ \ wbalanced s" using [[simp_depth_limit=1]] by(induction t arbitrary: s) auto -(* show wbalanced \ balanced and use that in Balanced.thy *) - subsection \@{const path_len}\