# HG changeset patch # User wenzelm # Date 1450736645 -3600 # Node ID f833208ff7c1ef9e806a3579fefd676d5df69695 # Parent e44d5b953f162620df1944ecd2cb7fae2bd5b533 dead code; diff -r e44d5b953f16 -r f833208ff7c1 src/HOL/Library/Sum_of_Squares_Remote.thy --- a/src/HOL/Library/Sum_of_Squares_Remote.thy Mon Dec 21 21:53:49 2015 +0100 +++ /dev/null Thu Jan 01 00:00:00 1970 +0000 @@ -1,36 +0,0 @@ -(* Title: HOL/Library/Sum_of_Squares_Remote.thy - Author: Amine Chaieb, University of Cambridge - Author: Philipp Meyer, TU Muenchen -*) - -section \Examples with remote CSDP\ - -theory Sum_of_Squares_Remote -imports Sum_of_Squares -begin - -lemma "(3::real) * x + 7 * a < 4 & 3 < 2 * x \ a < 0" - by (sos remote_csdp) - -lemma "a1 >= 0 & a2 >= 0 \ (a1 * a1 + a2 * a2 = b1 * b1 + b2 * b2 + 2) \ (a1 * b1 + a2 * b2 = 0) --> a1 * a2 - b1 * b2 >= (0::real)" - by (sos remote_csdp) - -lemma "(3::real) * x + 7 * a < 4 & 3 < 2 * x --> a < 0" - by (sos remote_csdp) - -lemma "(0::real) <= x & x <= 1 & 0 <= y & y <= 1 --> x^2 + y^2 < 1 |(x - 1)^2 + y^2 < 1 | x^2 + (y - 1)^2 < 1 | (x - 1)^2 + (y - 1)^2 < 1" - by (sos remote_csdp) - -lemma "(0::real) <= x & 0 <= y & 0 <= z & x + y + z <= 3 --> x * y + x * z + y * z >= 3 * x * y * z" - by (sos remote_csdp) - -lemma "((x::real)^2 + y^2 + z^2 = 1) --> (x + y + z)^2 <= 3" - by (sos remote_csdp) - -lemma "(w^2 + x^2 + y^2 + z^2 = 1) --> (w + x + y + z)^2 <= (4::real)" - by (sos remote_csdp) - -lemma "(x::real) >= 1 & y >= 1 --> x * y >= x + y - 1" - by (sos remote_csdp) - -end