| changeset 54864 | a064732223ad | 
| parent 53015 | a1119cf551e8 | 
| child 55465 | 0d31c0546286 | 
--- a/src/HOL/Metis_Examples/Binary_Tree.thy Wed Dec 25 17:39:06 2013 +0100 +++ b/src/HOL/Metis_Examples/Binary_Tree.thy Wed Dec 25 17:39:07 2013 +0100 @@ -80,7 +80,7 @@ lemma depth_reflect: "depth (reflect t) = depth t" apply (induct t) apply (metis depth.simps(1) reflect.simps(1)) -by (metis depth.simps(2) min_max.inf_sup_aci(5) reflect.simps(2)) +by (metis depth.simps(2) max.commute reflect.simps(2)) text {* The famous relationship between the numbers of leaves and nodes.