diff -r 2af982715e5c -r 03ce2b2a29a2 src/HOL/ex/Set_Theory.thy --- a/src/HOL/ex/Set_Theory.thy Sat Dec 24 15:53:09 2011 +0100 +++ b/src/HOL/ex/Set_Theory.thy Sat Dec 24 15:53:09 2011 +0100 @@ -179,7 +179,7 @@ lemma "a < b \ b < (c::int) \ \A. a \ A \ b \ A \ c \ A" -- {* Example 4. *} - by force + by auto --{*slow*} lemma "P (f b) \ \s A. (\x \ A. P x) \ f s \ A" -- {*Example 5, page 298. *} @@ -194,9 +194,9 @@ by force lemma "(\u v. u < (0::int) \ u \ abs v) - \ (\A::int set. (\y. abs y \ A) \ -2 \ A)" - -- {* Example 8 now needs a small hint. *} - by (simp add: abs_if, force) + \ (\A::int set. -2 \ A & (\y. abs y \ A))" + -- {* Example 8 needs a small hint. *} + by force -- {* not @{text blast}, which can't simplify @{text "-2 < 0"} *} text {* Example 9 omitted (requires the reals). *}