| changeset 45608 | 13b101cee425 |
| parent 44890 | 22f665a2e91c |
| child 45694 | 4a8743618257 |
--- a/src/HOL/Library/Multiset.thy Sun Nov 20 21:07:10 2011 +0100 +++ b/src/HOL/Library/Multiset.thy Sun Nov 20 21:28:07 2011 +0100 @@ -1527,7 +1527,7 @@ apply (rule iffI) prefer 2 apply blast -apply (rule_tac A=A and f=f in fold_msetG_nonempty [THEN exE, standard]) +apply (rule_tac A1=A and f1=f in fold_msetG_nonempty [THEN exE]) apply (blast intro: fold_msetG_determ) done