src/HOL/Algebra/Polynomials.thy
changeset 68582 b9b9e2985878
parent 68579 6dff90eba493
child 68584 ec4fe1032b6e
--- a/src/HOL/Algebra/Polynomials.thy	Tue Jul 03 10:49:44 2018 +0200
+++ b/src/HOL/Algebra/Polynomials.thy	Tue Jul 03 11:00:37 2018 +0200
@@ -1,11 +1,9 @@
-(* ************************************************************************** *)
-(* Title:      Polynomials.thy                                                *)
-(* Author:     Paulo Emílio de Vilhena                                        *)
-(* ************************************************************************** *)
+(*  Title:      HOL/Algebra/Polynomials.thy
+    Author:     Paulo Emílio de Vilhena
+*)
 
 theory Polynomials
   imports Ring Ring_Divisibility Subrings
-
 begin
 
 section \<open>Polynomials\<close>
@@ -1851,5 +1849,4 @@
          simp add: univ_poly_def degree_def
          simp del: poly_add.simps poly_mult.simps)
 
-
-end
\ No newline at end of file
+end