src/HOL/Library/Permutation.thy
changeset 14706 71590b7733b7
parent 11153 950ede59c05a
child 15005 546c8e7e28d4
--- a/src/HOL/Library/Permutation.thy	Thu May 06 12:43:00 2004 +0200
+++ b/src/HOL/Library/Permutation.thy	Thu May 06 14:14:18 2004 +0200
@@ -1,16 +1,13 @@
 (*  Title:      HOL/Library/Permutation.thy
     ID:         $Id$
-    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
+    Author:     Lawrence C Paulson and Thomas M Rasmussen
     Copyright   1995  University of Cambridge
 
 TODO: it would be nice to prove (for "multiset", defined on
 HOL/ex/Sorting.thy) xs <~~> ys = (\<forall>x. multiset xs x = multiset ys x)
 *)
 
-header {*
- \title{Permutations}
- \author{Lawrence C Paulson and Thomas M Rasmussen}
-*}
+header {* Permutations *}
 
 theory Permutation = Main: