diff -r 863258b0cdca -r 3676def6b8b9 src/HOL/ex/Refute_Examples.thy --- a/src/HOL/ex/Refute_Examples.thy Fri Mar 26 14:53:17 2004 +0100 +++ b/src/HOL/ex/Refute_Examples.thy Fri Mar 26 19:58:43 2004 +0100 @@ -26,7 +26,7 @@ refute [satsolver="dpll"] 2 -- {* ... and specify a subgoal at the same time *} oops -refute_params +refute_params [satsolver="dpll"] section {* Examples and Test Cases *} @@ -155,7 +155,7 @@ text {* A true statement (also testing names of free and bound variables being identical) *} lemma "(\x y. P x y \ P y x) \ (\x. P x y) \ P y x" - refute [maxsize=2] (* [maxsize=5] works well with ZChaff *) + refute apply fast done @@ -172,13 +172,13 @@ text {* "Every reflexive and symmetric relation is transitive." *} lemma "\ \x. P x x; \x y. P x y \ P y x \ \ P x y \ P y z \ P x z" - (* refute -- works well with ZChaff, but the internal solver is too slow *) + refute oops text {* The "Drinker's theorem" ... *} lemma "\x. f x = g x \ f = g" - refute [maxsize=4] (* [maxsize=6] works well with ZChaff *) + refute apply (auto simp add: ext) done @@ -262,7 +262,7 @@ \ trans_closure TP P \ trans_closure TR R \ (T x y = (TP x y | TR x y))" - (* refute -- works well with ZChaff, but the internal solver is too slow *) + refute oops text {* "Every surjective function is invertible." *} @@ -280,7 +280,7 @@ text {* Every point is a fixed point of some function. *} lemma "\f. f x = x" - refute [maxsize=4] + refute [maxsize=5] apply (rule_tac x="\x. x" in exI) apply simp done @@ -294,12 +294,12 @@ text {* ... and now two correct ones *} lemma "(\x. \y. P x y) \ (\f. \x. P x (f x))" - refute [maxsize=5] + refute apply (simp add: choice) done lemma "(\x. EX!y. P x y) \ (EX!f. \x. P x (f x))" - refute [maxsize=3] (* [maxsize=4] works well with ZChaff *) + refute apply auto apply (simp add: ex1_implies_ex choice) apply (fast intro: ext) @@ -361,7 +361,7 @@ oops lemma "{x. P x} = {y. P y}" - refute [maxsize=2] (* [maxsize=8] works well with ZChaff *) + refute apply simp done @@ -430,7 +430,7 @@ oops lemma "Ex P \ P (The P)" - (* refute -- works well with ZChaff, but the internal solver is too slow *) + refute oops subsection {* Eps *} @@ -452,7 +452,7 @@ oops lemma "Ex P \ P (Eps P)" - refute [maxsize=2] (* [maxsize=3] works well with ZChaff *) + refute [maxsize=3] apply (auto simp add: someI) done