| changeset 64242 | 93c6f0da5c70 |
| parent 63411 | e051eea34990 |
| child 64947 | f6ad52152040 |
--- a/src/HOL/Data_Structures/RBT_Set.thy Sun Oct 16 09:31:04 2016 +0200 +++ b/src/HOL/Data_Structures/RBT_Set.thy Sun Oct 16 09:31:05 2016 +0200 @@ -419,7 +419,7 @@ next case (2 h t t') with RB_mod obtain n where "2*n + 1 = h" - by (metis color.distinct(1) mod_div_equality2 parity) + by (metis color.distinct(1) mult_div_mod_eq parity) with 2 balB_h RB_h show ?case by auto next case (3 h t t')