src/HOL/ex/set.thy
changeset 14353 79f9fbef9106
parent 13107 8743cc847224
child 15306 51f3d31e8eea
--- a/src/HOL/ex/set.thy	Mon Jan 12 16:45:35 2004 +0100
+++ b/src/HOL/ex/set.thy	Mon Jan 12 16:51:45 2004 +0100
@@ -156,8 +156,9 @@
 
 lemma "(\<forall>u v. u < (0::int) \<longrightarrow> u \<noteq> abs v)
     \<longrightarrow> (\<exists>A::int set. (\<forall>y. abs y \<notin> A) \<and> -2 \<in> A)"
-  -- {* Example 8. *}
-  by force  -- {* not @{text blast}, which can't simplify @{text "-2 < 0"} *}
+  -- {* Example 8 now needs a small hint. *}
+  by (simp add: abs_if, force)
+    -- {* not @{text blast}, which can't simplify @{text "-2 < 0"} *}
 
 text {* Example 9 omitted (requires the reals). *}