tuned headers;
authorwenzelm
Fri, 07 Apr 2017 21:17:18 +0200
changeset 65435 378175f44328
parent 65434 e62b1af601f0
child 65436 1fd2dca8eb60
child 65437 b8fc7e2e1b35
child 65439 862bfd2b4fd4
tuned headers;
src/HOL/Algebra/More_Ring.thy
src/HOL/Computational_Algebra/Euclidean_Algorithm.thy
src/HOL/Computational_Algebra/Factorial_Ring.thy
src/HOL/Computational_Algebra/Field_as_Ring.thy
src/HOL/Computational_Algebra/Formal_Power_Series.thy
src/HOL/Computational_Algebra/Fraction_Field.thy
src/HOL/Computational_Algebra/Fundamental_Theorem_Algebra.thy
src/HOL/Computational_Algebra/Normalized_Fraction.thy
src/HOL/Computational_Algebra/Polynomial.thy
src/HOL/Computational_Algebra/Polynomial_FPS.thy
src/HOL/Computational_Algebra/Polynomial_Factorial.thy
src/HOL/Computational_Algebra/Primes.thy
src/HOL/Number_Theory/Gauss.thy
--- a/src/HOL/Algebra/More_Ring.thy	Fri Apr 07 21:07:07 2017 +0200
+++ b/src/HOL/Algebra/More_Ring.thy	Fri Apr 07 21:17:18 2017 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/Algebra/More_Group.thy
+(*  Title:      HOL/Algebra/More_Ring.thy
     Author:     Jeremy Avigad
 *)
 
--- a/src/HOL/Computational_Algebra/Euclidean_Algorithm.thy	Fri Apr 07 21:07:07 2017 +0200
+++ b/src/HOL/Computational_Algebra/Euclidean_Algorithm.thy	Fri Apr 07 21:17:18 2017 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/Number_Theory/Euclidean_Algorithm.thy
+(*  Title:      HOL/Computational_Algebra/Euclidean_Algorithm.thy
     Author:     Manuel Eberl, TU Muenchen
 *)
 
--- a/src/HOL/Computational_Algebra/Factorial_Ring.thy	Fri Apr 07 21:07:07 2017 +0200
+++ b/src/HOL/Computational_Algebra/Factorial_Ring.thy	Fri Apr 07 21:17:18 2017 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/Number_Theory/Factorial_Ring.thy
+(*  Title:      HOL/Computational_Algebra/Factorial_Ring.thy
     Author:     Manuel Eberl, TU Muenchen
     Author:     Florian Haftmann, TU Muenchen
 *)
--- a/src/HOL/Computational_Algebra/Field_as_Ring.thy	Fri Apr 07 21:07:07 2017 +0200
+++ b/src/HOL/Computational_Algebra/Field_as_Ring.thy	Fri Apr 07 21:17:18 2017 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/Library/Field_as_Ring.thy
+(*  Title:      HOL/Computational_Algebra/Field_as_Ring.thy
     Author:     Manuel Eberl
 *)
 
--- a/src/HOL/Computational_Algebra/Formal_Power_Series.thy	Fri Apr 07 21:07:07 2017 +0200
+++ b/src/HOL/Computational_Algebra/Formal_Power_Series.thy	Fri Apr 07 21:17:18 2017 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/Library/Formal_Power_Series.thy
+(*  Title:      HOL/Computational_Algebra/Formal_Power_Series.thy
     Author:     Amine Chaieb, University of Cambridge
 *)
 
--- a/src/HOL/Computational_Algebra/Fraction_Field.thy	Fri Apr 07 21:07:07 2017 +0200
+++ b/src/HOL/Computational_Algebra/Fraction_Field.thy	Fri Apr 07 21:17:18 2017 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/Library/Fraction_Field.thy
+(*  Title:      HOL/Computational_Algebra/Fraction_Field.thy
     Author:     Amine Chaieb, University of Cambridge
 *)
 
--- a/src/HOL/Computational_Algebra/Fundamental_Theorem_Algebra.thy	Fri Apr 07 21:07:07 2017 +0200
+++ b/src/HOL/Computational_Algebra/Fundamental_Theorem_Algebra.thy	Fri Apr 07 21:17:18 2017 +0200
@@ -1,4 +1,6 @@
-(* Author: Amine Chaieb, TU Muenchen *)
+(*  Title:      HOL/Computational_Algebra/Fundamental_Theorem_Algebra.thy
+    Author:     Amine Chaieb, TU Muenchen
+*)
 
 section \<open>Fundamental Theorem of Algebra\<close>
 
--- a/src/HOL/Computational_Algebra/Normalized_Fraction.thy	Fri Apr 07 21:07:07 2017 +0200
+++ b/src/HOL/Computational_Algebra/Normalized_Fraction.thy	Fri Apr 07 21:17:18 2017 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/Library/Normalized_Fraction.thy
+(*  Title:      HOL/Computational_Algebra/Normalized_Fraction.thy
     Author:     Manuel Eberl
 *)
 
--- a/src/HOL/Computational_Algebra/Polynomial.thy	Fri Apr 07 21:07:07 2017 +0200
+++ b/src/HOL/Computational_Algebra/Polynomial.thy	Fri Apr 07 21:17:18 2017 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/Library/Polynomial.thy
+(*  Title:      HOL/Computational_Algebra/Polynomial.thy
     Author:     Brian Huffman
     Author:     Clemens Ballarin
     Author:     Amine Chaieb
--- a/src/HOL/Computational_Algebra/Polynomial_FPS.thy	Fri Apr 07 21:07:07 2017 +0200
+++ b/src/HOL/Computational_Algebra/Polynomial_FPS.thy	Fri Apr 07 21:17:18 2017 +0200
@@ -1,7 +1,5 @@
-(*  Title:      HOL/Library/Polynomial_FPS.thy
+(*  Title:      HOL/Computational_Algebra/Polynomial_FPS.thy
     Author:     Manuel Eberl, TU München
-  
-Converting polynomials to formal power series.
 *)
 
 section \<open>Converting polynomials to formal power series\<close>
--- a/src/HOL/Computational_Algebra/Polynomial_Factorial.thy	Fri Apr 07 21:07:07 2017 +0200
+++ b/src/HOL/Computational_Algebra/Polynomial_Factorial.thy	Fri Apr 07 21:17:18 2017 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/Library/Polynomial_Factorial.thy
+(*  Title:      HOL/Computational_Algebra/Polynomial_Factorial.thy
     Author:     Brian Huffman
     Author:     Clemens Ballarin
     Author:     Amine Chaieb
--- 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
--- a/src/HOL/Number_Theory/Gauss.thy	Fri Apr 07 21:07:07 2017 +0200
+++ b/src/HOL/Number_Theory/Gauss.thy	Fri Apr 07 21:17:18 2017 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/Number_Theory/Quadratic_Reciprocity.thy
+(*  Title:      HOL/Number_Theory/Gauss.thy
     Authors:    Jeremy Avigad, David Gray, and Adam Kramer
 
 Ported by lcp but unfinished.