diff -r 2c357e2b8436 -r ade3fc826af3 src/HOL/SMT_Examples/SMT_Tests.thy --- a/src/HOL/SMT_Examples/SMT_Tests.thy Tue Mar 27 16:59:13 2012 +0300 +++ b/src/HOL/SMT_Examples/SMT_Tests.thy Tue Mar 27 17:11:02 2012 +0200 @@ -104,18 +104,6 @@ by smt+ lemma - "distinct []" - "distinct [a]" - "distinct [a, b, c] \ a \ c" - "distinct [a, b, c] \ d = b \ a \ d" - "\ distinct [a, b, a, b]" - "a = b \ \ distinct [a, b]" - "a = b \ a = c \ \ distinct [a, b, c]" - "distinct [a, b, c, d] \ distinct [d, b, c, a]" - "distinct [a, b, c, d] \ distinct [a, b, c] \ distinct [b, c, d]" - by smt+ - -lemma "\x. x = x" "(\x. P x) \ (\y. P y)" "\x. P x \ (\y. P x \ P y)" @@ -193,7 +181,7 @@ by smt+ lemma - "distinct [a, b, c] \ (\x y. f x = f y \ y = x) \ f a \ f b" + "a \ b \ a \ c \ b \ c \ (\x y. f x = f y \ y = x) \ f a \ f b" by smt lemma @@ -932,7 +920,7 @@ "i1 \ i2 \ (f (i1 := v1, i2 := v2)) i2 = v2" "i1 = i2 \ (f (i1 := v1, i2 := v2)) i1 = v2" "i1 = i2 \ (f (i1 := v1, i2 := v2)) i1 = v2" - "distinct [i1, i2, i3] \ (f (i1 := v1, i2 := v2)) i3 = f i3" + "i1 \ i2 \i1 \ i3 \ i2 \ i3 \ (f (i1 := v1, i2 := v2)) i3 = f i3" using fun_upd_same fun_upd_apply by smt+