| changeset 33059 | d1c9bf0f8ae8 |
| parent 33057 | 764547b68538 |
| child 33715 | 8cce3a34c122 |
--- a/src/HOL/Library/Permutations.thy Thu Oct 22 09:49:48 2009 +0200 +++ b/src/HOL/Library/Permutations.thy Thu Oct 22 09:50:29 2009 +0200 @@ -83,7 +83,7 @@ unfolding permutes_def by simp lemma permutes_inv_eq: "p permutes S ==> inv p y = x \<longleftrightarrow> p x = y" - unfolding permutes_def inv_onto_def apply auto + unfolding permutes_def inv_def apply auto apply (erule allE[where x=y]) apply (erule allE[where x=y]) apply (rule someI_ex) apply blast