diff -r f38b94549dc8 -r fbe93138e540 src/HOL/ex/Refute_Examples.thy --- a/src/HOL/ex/Refute_Examples.thy Thu Apr 09 18:00:58 2015 +0200 +++ b/src/HOL/ex/Refute_Examples.thy Thu Apr 09 18:00:59 2015 +0200 @@ -259,15 +259,6 @@ refute [expect = genuine] oops -text {* "The union of transitive closures is equal to the transitive closure of unions." *} - -lemma "(\x y. (P x y | R x y) \ T x y) \ trans T \ (\Q. (\x y. (P x y | R x y) \ Q x y) \ trans Q \ subset T Q) - \ trans_closure TP P - \ trans_closure TR R - \ (T x y = (TP x y | TR x y))" -refute [expect = genuine] -oops - text {* "Every surjective function is invertible." *} lemma "(\y. \x. y = f x) \ (\g. \x. g (f x) = x)"