# HG changeset patch # User wenzelm # Date 1426521599 -3600 # Node ID f893472fff31ee1a3bcef3df697b33849fb6fe2e # Parent 6410a310fdc2ec77b77bf73b057a09a1b92b9168 proper headers; diff -r 6410a310fdc2 -r f893472fff31 src/Doc/Logics_ZF/If.thy --- a/src/Doc/Logics_ZF/If.thy Mon Mar 16 16:26:33 2015 +0100 +++ b/src/Doc/Logics_ZF/If.thy Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -(* Title: Doc/ZF/If.thy +(* Title: Doc/Logics_ZF/If.thy Author: Lawrence C Paulson, Cambridge University Computer Laboratory Copyright 1991 University of Cambridge diff -r 6410a310fdc2 -r f893472fff31 src/HOL/Codegenerator_Test/Code_Test_GHC.thy --- a/src/HOL/Codegenerator_Test/Code_Test_GHC.thy Mon Mar 16 16:26:33 2015 +0100 +++ b/src/HOL/Codegenerator_Test/Code_Test_GHC.thy Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -(* Title: Code_Test_GHC.thy +(* Title: HOL/Codegenerator_Test/Code_Test_GHC.thy Author: Andreas Lochbihler, ETH Zurich Test case for test_code on GHC diff -r 6410a310fdc2 -r f893472fff31 src/HOL/Codegenerator_Test/Code_Test_MLton.thy --- a/src/HOL/Codegenerator_Test/Code_Test_MLton.thy Mon Mar 16 16:26:33 2015 +0100 +++ b/src/HOL/Codegenerator_Test/Code_Test_MLton.thy Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -(* Title: Code_Test_MLtonL.thy +(* Title: HOL/Codegenerator_Test/Code_Test_MLton.thy Author: Andreas Lochbihler, ETH Zurich Test case for test_code on MLton diff -r 6410a310fdc2 -r f893472fff31 src/HOL/Codegenerator_Test/Code_Test_OCaml.thy --- a/src/HOL/Codegenerator_Test/Code_Test_OCaml.thy Mon Mar 16 16:26:33 2015 +0100 +++ b/src/HOL/Codegenerator_Test/Code_Test_OCaml.thy Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -(* Title: Code_Test_OCaml.thy +(* Title: HOL/Codegenerator_Test/Code_Test_OCaml.thy Author: Andreas Lochbihler, ETH Zurich Test case for test_code on OCaml diff -r 6410a310fdc2 -r f893472fff31 src/HOL/Codegenerator_Test/Code_Test_PolyML.thy --- a/src/HOL/Codegenerator_Test/Code_Test_PolyML.thy Mon Mar 16 16:26:33 2015 +0100 +++ b/src/HOL/Codegenerator_Test/Code_Test_PolyML.thy Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -(* Title: Code_Test_PolyML.thy +(* Title: HOL/Codegenerator_Test/Code_Test_PolyML.thy Author: Andreas Lochbihler, ETH Zurich Test case for test_code on PolyML diff -r 6410a310fdc2 -r f893472fff31 src/HOL/Codegenerator_Test/Code_Test_SMLNJ.thy --- a/src/HOL/Codegenerator_Test/Code_Test_SMLNJ.thy Mon Mar 16 16:26:33 2015 +0100 +++ b/src/HOL/Codegenerator_Test/Code_Test_SMLNJ.thy Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -(* Title: Code_Test_SMLNJ.thy +(* Title: HOL/Codegenerator_Test/Code_Test_SMLNJ.thy Author: Andreas Lochbihler, ETH Zurich Test case for test_code on SMLNJ diff -r 6410a310fdc2 -r f893472fff31 src/HOL/Codegenerator_Test/Code_Test_Scala.thy --- a/src/HOL/Codegenerator_Test/Code_Test_Scala.thy Mon Mar 16 16:26:33 2015 +0100 +++ b/src/HOL/Codegenerator_Test/Code_Test_Scala.thy Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -(* Title: Code_Test_Scala.thy +(* Title: HOL/Codegenerator_Test/Code_Test_Scala.thy Author: Andreas Lochbihler, ETH Zurich Test case for test_code on Scala diff -r 6410a310fdc2 -r f893472fff31 src/HOL/Inequalities.thy --- a/src/HOL/Inequalities.thy Mon Mar 16 16:26:33 2015 +0100 +++ b/src/HOL/Inequalities.thy Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -(* Title: Inequalities +(* Title: HOL/Inequalities.thy Author: Tobias Nipkow Author: Johannes Hölzl *) diff -r 6410a310fdc2 -r f893472fff31 src/HOL/Library/Code_Test.thy --- a/src/HOL/Library/Code_Test.thy Mon Mar 16 16:26:33 2015 +0100 +++ b/src/HOL/Library/Code_Test.thy Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -(* Title: Code_Test.thy +(* Title: HOL/Library/Code_Test.thy Author: Andreas Lochbihler, ETH Zurich Test infrastructure for the code generator diff -r 6410a310fdc2 -r f893472fff31 src/HOL/Library/ContNotDenum.thy --- a/src/HOL/Library/ContNotDenum.thy Mon Mar 16 16:26:33 2015 +0100 +++ b/src/HOL/Library/ContNotDenum.thy Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -(* Title: HOL/Library/ContNonDenum.thy +(* Title: HOL/Library/ContNotDenum.thy Author: Benjamin Porter, Monash University, NICTA, 2005 Author: Johannes Hölzl, TU München *) diff -r 6410a310fdc2 -r f893472fff31 src/HOL/Library/code_test.ML --- a/src/HOL/Library/code_test.ML Mon Mar 16 16:26:33 2015 +0100 +++ b/src/HOL/Library/code_test.ML Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -(* Title: Code_Test.ML +(* Title: HOL/Library/code_test.ML Author: Andreas Lochbihler, ETH Zurich Test infrastructure for the code generator diff -r 6410a310fdc2 -r f893472fff31 src/HOL/TPTP/TPTP_Proof_Reconstruction_Test.thy --- a/src/HOL/TPTP/TPTP_Proof_Reconstruction_Test.thy Mon Mar 16 16:26:33 2015 +0100 +++ b/src/HOL/TPTP/TPTP_Proof_Reconstruction_Test.thy Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -(* Title: HOL/TPTP/TPTP_Proof_Reconstruction.thy +(* Title: HOL/TPTP/TPTP_Proof_Reconstruction_Test.thy Author: Nik Sultana, Cambridge University Computer Laboratory Various tests for the proof reconstruction module. diff -r 6410a310fdc2 -r f893472fff31 src/HOL/TPTP/TPTP_Proof_Reconstruction_Test_Units.thy --- a/src/HOL/TPTP/TPTP_Proof_Reconstruction_Test_Units.thy Mon Mar 16 16:26:33 2015 +0100 +++ b/src/HOL/TPTP/TPTP_Proof_Reconstruction_Test_Units.thy Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -(* Title: HOL/TPTP/TPTP_Proof_Reconstruction.thy +(* Title: HOL/TPTP/TPTP_Proof_Reconstruction_Test_Units.thy Author: Nik Sultana, Cambridge University Computer Laboratory Unit tests for proof reconstruction module. diff -r 6410a310fdc2 -r f893472fff31 src/HOL/Tools/Lifting/lifting_bnf.ML --- a/src/HOL/Tools/Lifting/lifting_bnf.ML Mon Mar 16 16:26:33 2015 +0100 +++ b/src/HOL/Tools/Lifting/lifting_bnf.ML Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -(* Title: HOL/Tools/Transfer/transfer_bnf.ML +(* Title: HOL/Tools/Lifting/lifting_bnf.ML Author: Ondrej Kuncar, TU Muenchen Setup for Lifting for types that are BNF. diff -r 6410a310fdc2 -r f893472fff31 src/Pure/Concurrent/random.ML --- a/src/Pure/Concurrent/random.ML Mon Mar 16 16:26:33 2015 +0100 +++ b/src/Pure/Concurrent/random.ML Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -(* Title: Pure/Confurrent/random.ML +(* Title: Pure/Concurrent/random.ML Author: Lawrence C Paulson, Cambridge University Computer Laboratory Pseudo random numbers. diff -r 6410a310fdc2 -r f893472fff31 src/Pure/GUI/jfx_gui.scala --- a/src/Pure/GUI/jfx_gui.scala Mon Mar 16 16:26:33 2015 +0100 +++ b/src/Pure/GUI/jfx_gui.scala Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -/* Title: Pure/GUI/jfx_thread.scala +/* Title: Pure/GUI/jfx_gui.scala Module: PIDE-JFX Author: Makarius diff -r 6410a310fdc2 -r f893472fff31 src/Pure/General/antiquote.scala --- a/src/Pure/General/antiquote.scala Mon Mar 16 16:26:33 2015 +0100 +++ b/src/Pure/General/antiquote.scala Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -/* Title: Pure/ML/antiquote.scala +/* Title: Pure/General/antiquote.scala Author: Makarius Antiquotations within plain text. diff -r 6410a310fdc2 -r f893472fff31 src/Pure/General/completion.ML --- a/src/Pure/General/completion.ML Mon Mar 16 16:26:33 2015 +0100 +++ b/src/Pure/General/completion.ML Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -(* Title: Pure/Isar/completion.ML +(* Title: Pure/General/completion.ML Author: Makarius Semantic completion within the formal context. diff -r 6410a310fdc2 -r f893472fff31 src/Pure/PIDE/batch_session.scala --- a/src/Pure/PIDE/batch_session.scala Mon Mar 16 16:26:33 2015 +0100 +++ b/src/Pure/PIDE/batch_session.scala Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -/* Title: Pure/Tools/batch_session.scala +/* Title: Pure/PIDE/batch_session.scala Author: Makarius PIDE session in batch mode. diff -r 6410a310fdc2 -r f893472fff31 src/Pure/System/posix_interrupt.scala --- a/src/Pure/System/posix_interrupt.scala Mon Mar 16 16:26:33 2015 +0100 +++ b/src/Pure/System/posix_interrupt.scala Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -/* Title: Pure/System/interrupt.scala +/* Title: Pure/System/posix_interrupt.scala Author: Makarius Support for POSIX interrupts (bypassed on Windows). diff -r 6410a310fdc2 -r f893472fff31 src/Pure/Tools/print_operation.scala --- a/src/Pure/Tools/print_operation.scala Mon Mar 16 16:26:33 2015 +0100 +++ b/src/Pure/Tools/print_operation.scala Mon Mar 16 16:59:59 2015 +0100 @@ -1,4 +1,4 @@ -/* Title: Pure/System/print_operation.scala +/* Title: Pure/Tools/print_operation.scala Author: Makarius Print operations as asynchronous query.