| changeset 46752 | e9e7209eb375 | 
| parent 45966 | 03ce2b2a29a2 | 
| child 58889 | 5b7a9633cfa8 | 
--- a/src/HOL/ex/Set_Theory.thy Thu Mar 01 17:13:54 2012 +0000 +++ b/src/HOL/ex/Set_Theory.thy Thu Mar 01 19:34:52 2012 +0100 @@ -128,7 +128,7 @@ let ?n = "card A" have "finite A" using `card A \<ge> 2` by(auto intro:ccontr) have 0: "R `` A <= A" using `sym R` `Domain R <= A` - unfolding Domain_def sym_def by blast + unfolding Domain_unfold sym_def by blast have h: "ALL a:A. R `` {a} <= A" using 0 by blast hence 1: "ALL a:A. finite(R `` {a})" using `finite A` by(blast intro: finite_subset)