src/HOL/Computational_Algebra/Primes.thy
changeset 65435 378175f44328
parent 65417 fc41a5650fb1
child 65583 8d53b3bebab4
--- a/src/HOL/Computational_Algebra/Primes.thy	Fri Apr 07 21:07:07 2017 +0200
+++ b/src/HOL/Computational_Algebra/Primes.thy	Fri Apr 07 21:17:18 2017 +0200
@@ -1,9 +1,13 @@
-(*  Authors:    Christophe Tabacznyj, Lawrence C. Paulson, Amine Chaieb,
-                Thomas M. Rasmussen, Jeremy Avigad, Tobias Nipkow, 
-                Manuel Eberl
+(*  Title:      HOL/Computational_Algebra/Primes.thy
+    Author:     Christophe Tabacznyj
+    Author:     Lawrence C. Paulson
+    Author:     Amine Chaieb
+    Author:     Thomas M. Rasmussen
+    Author:     Jeremy Avigad
+    Author:     Tobias Nipkow
+    Author:     Manuel Eberl
 
-
-This file deals with properties of primes. Definitions and lemmas are
+This theory deals with properties of primes. Definitions and lemmas are
 proved uniformly for the natural numbers and integers.
 
 This file combines and revises a number of prior developments.
@@ -32,7 +36,6 @@
 Thomas Marthedal Rasmussen, Jeremy Avigad, and David Gray.
 *)
 
-
 section \<open>Primes\<close>
 
 theory Primes