src/HOL/Algebra/Cycles.thy
changeset 68582 b9b9e2985878
parent 68569 c64319959bab
child 68605 440aa6b7d99a
--- a/src/HOL/Algebra/Cycles.thy	Tue Jul 03 10:49:44 2018 +0200
+++ b/src/HOL/Algebra/Cycles.thy	Tue Jul 03 11:00:37 2018 +0200
@@ -1,11 +1,9 @@
-(* ************************************************************************** *)
-(* Title:      Cycles.thy                                                     *)
-(* Author:     Paulo Emílio de Vilhena                                        *)
-(* ************************************************************************** *)
+(*  Title:      HOL/Algebra/Cycles.thy
+    Author:     Paulo Emílio de Vilhena
+*)
 
 theory Cycles
   imports "HOL-Library.Permutations" "HOL-Library.FuncSet"
-    
 begin
 
 section \<open>Cycles\<close>
@@ -753,4 +751,4 @@
   shows "cycle_decomp S p"
   using assms cycle_decomposition_aux by blast
 
-end
\ No newline at end of file
+end