diff -r 5d06ecfdb472 -r 1135b8de26c3 src/HOL/SMT_Examples/SMT_Tests.thy --- a/src/HOL/SMT_Examples/SMT_Tests.thy Mon Dec 28 01:26:34 2015 +0100 +++ b/src/HOL/SMT_Examples/SMT_Tests.thy Mon Dec 28 01:28:28 2015 +0100 @@ -336,11 +336,11 @@ by smt+ lemma - "abs (x::int) \ 0" - "(abs x = 0) = (x = 0)" - "(x \ 0) = (abs x = x)" - "(x \ 0) = (abs x = -x)" - "abs (abs x) = abs x" + "\x::int\ \ 0" + "(\x\ = 0) = (x = 0)" + "(x \ 0) = (\x\ = x)" + "(x \ 0) = (\x\ = -x)" + "\\x\\ = \x\" by smt+ lemma @@ -349,7 +349,7 @@ "z < x \ z < y \ z < min x y" "min x y = min y x" "x \ 0 \ min x 0 = 0" - "min x y \ abs (x + y)" + "min x y \ \x + y\" by smt+ lemma @@ -358,7 +358,7 @@ "z > x \ z > y \ z > max x y" "max x y = max y x" "x \ 0 \ max x 0 = x" - "max x y \ - abs x - abs y" + "max x y \ - \x\ - \y\" by smt+ lemma @@ -448,11 +448,11 @@ by smt+ lemma - "abs (x::real) \ 0" - "(abs x = 0) = (x = 0)" - "(x \ 0) = (abs x = x)" - "(x \ 0) = (abs x = -x)" - "abs (abs x) = abs x" + "\x::real\ \ 0" + "(\x\ = 0) = (x = 0)" + "(x \ 0) = (\x\ = x)" + "(x \ 0) = (\x\ = -x)" + "\\x\\ = \x\" by smt+ lemma @@ -461,7 +461,7 @@ "z < x \ z < y \ z < min x y" "min x y = min y x" "x \ 0 \ min x 0 = 0" - "min x y \ abs (x + y)" + "min x y \ \x + y\" by smt+ lemma @@ -470,7 +470,7 @@ "z > x \ z > y \ z > max x y" "max x y = max y x" "x \ 0 \ max x 0 = x" - "max x y \ - abs x - abs y" + "max x y \ - \x\ - \y\" by smt+ lemma