src/HOL/ex/SOS_Remote.thy
changeset 58636 9b33fe5b60f3
parent 58627 1329679abb2d
parent 58635 010b610eb55d
child 58637 3094b0edd6b5
child 58638 5855b9b3d6a3
--- a/src/HOL/ex/SOS_Remote.thy	Wed Oct 08 10:22:00 2014 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,37 +0,0 @@
-(*  Title:      HOL/ex/SOS_Remote.thy
-    Author:     Amine Chaieb, University of Cambridge
-    Author:     Philipp Meyer, TU Muenchen
-
-Examples for Sum_of_Squares: remote CSDP server.
-*)
-
-theory SOS_Remote
-imports "~~/src/HOL/Library/Sum_of_Squares"
-begin
-
-lemma "(3::real) * x + 7 * a < 4 & 3 < 2 * x \<Longrightarrow> a < 0"
-  by (sos remote_csdp)
-
-lemma "a1 >= 0 & a2 >= 0 \<and> (a1 * a1 + a2 * a2 = b1 * b1 + b2 * b2 + 2) \<and> (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
-