diff -r 28cd3c9ca278 -r fb696ff1f086 src/HOL/Wellfounded.thy --- a/src/HOL/Wellfounded.thy Sat Oct 20 09:09:33 2012 +0200 +++ b/src/HOL/Wellfounded.thy Sat Oct 20 09:09:34 2012 +0200 @@ -764,9 +764,9 @@ with Mw show "?N2 \ ?W" by (simp only:) next assume "M \ {}" - have N2: "(?N2, M) \ max_ext r" - by (rule max_extI[OF _ _ `M \ {}`]) (insert asm1, auto intro: finites) - + from asm1 finites have N2: "(?N2, M) \ max_ext r" + by (rule_tac max_extI[OF _ _ `M \ {}`]) auto + with `M \ ?W` show "?N2 \ ?W" by (rule acc_downward) qed with finites have "?N1 \ ?N2 \ ?W"