src/HOL/Library/Sum_Of_Squares.thy
changeset 32949 aa6c470a962a
parent 32645 1cc5b24f5a01
child 33041 6793b02a3409
--- a/src/HOL/Library/Sum_Of_Squares.thy	Thu Oct 15 17:49:30 2009 +0200
+++ b/src/HOL/Library/Sum_Of_Squares.thy	Thu Oct 15 21:08:03 2009 +0200
@@ -1,5 +1,6 @@
-(* Title:      HOL/Library/Sum_Of_Squares.thy
-   Author:     Amine Chaieb, University of Cambridge
+(*  Title:      HOL/Library/Sum_Of_Squares.thy
+    Author:     Amine Chaieb, University of Cambridge
+    Author:     Philipp Meyer, TU Muenchen
 *)
 
 header {* A decision method for universal multivariate real arithmetic with addition, 
@@ -34,7 +35,7 @@
 use "Sum_Of_Squares/sum_of_squares.ML"
 use "Sum_Of_Squares/sos_wrapper.ML"
 
-setup SosWrapper.setup
+setup SOS_Wrapper.setup
 
 text {* Tests *}