tuned headers;
authorwenzelm
Thu, 30 May 2013 23:29:33 +0200
changeset 52265 bb907eba5902
parent 52264 cdba0c3cb4c2
child 52266 86d6f57c2c1e
child 52267 2a16957cd379
tuned headers;
src/HOL/Conditionally_Complete_Lattices.thy
src/HOL/Limits.thy
src/HOL/Tools/case_translation.ML
src/HOL/Topological_Spaces.thy
src/Tools/Code/code_symbol.ML
--- a/src/HOL/Conditionally_Complete_Lattices.thy	Thu May 30 22:30:38 2013 +0200
+++ b/src/HOL/Conditionally_Complete_Lattices.thy	Thu May 30 23:29:33 2013 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/Conditional_Complete_Lattices.thy
+(*  Title:      HOL/Conditionally_Complete_Lattices.thy
     Author:     Amine Chaieb and L C Paulson, University of Cambridge
     Author:     Johannes Hölzl, TU München
 *)
--- a/src/HOL/Limits.thy	Thu May 30 22:30:38 2013 +0200
+++ b/src/HOL/Limits.thy	Thu May 30 23:29:33 2013 +0200
@@ -1,4 +1,4 @@
-(*  Title:      Limits.thy
+(*  Title:      HOL/Limits.thy
     Author:     Brian Huffman
     Author:     Jacques D. Fleuriot, University of Cambridge
     Author:     Lawrence C Paulson
--- a/src/HOL/Tools/case_translation.ML	Thu May 30 22:30:38 2013 +0200
+++ b/src/HOL/Tools/case_translation.ML	Thu May 30 23:29:33 2013 +0200
@@ -1,4 +1,4 @@
-(*  Title:      Tools/case_translation.ML
+(*  Title:      HOL/Tools/case_translation.ML
     Author:     Konrad Slind, Cambridge University Computer Laboratory
     Author:     Stefan Berghofer, TU Muenchen
     Author:     Dmitriy Traytel, TU Muenchen
--- a/src/HOL/Topological_Spaces.thy	Thu May 30 22:30:38 2013 +0200
+++ b/src/HOL/Topological_Spaces.thy	Thu May 30 23:29:33 2013 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/Basic_Topology.thy
+(*  Title:      HOL/Topological_Spaces.thy
     Author:     Brian Huffman
     Author:     Johannes Hölzl
 *)
--- a/src/Tools/Code/code_symbol.ML	Thu May 30 22:30:38 2013 +0200
+++ b/src/Tools/Code/code_symbol.ML	Thu May 30 23:29:33 2013 +0200
@@ -1,4 +1,4 @@
-(*  Title:      Tools/Code/ML
+(*  Title:      Tools/Code/code_symbol.ML
     Author:     Florian Haftmann, TU Muenchen
 
 Data related to symbols in programs: constants, type constructors, classes,