tuned comments;
authorwenzelm
Wed, 13 Jun 2007 18:30:15 +0200
changeset 23374 a2f492c599e0
parent 23373 ead82c82da9e
child 23375 45cd7db985b3
tuned comments;
src/HOL/Library/SCT_Definition.thy
src/HOL/Library/SCT_Examples.thy
src/HOL/Library/SCT_Implementation.thy
src/HOL/Library/SCT_Interpretation.thy
src/HOL/Library/Size_Change_Termination.thy
--- a/src/HOL/Library/SCT_Definition.thy	Wed Jun 13 18:30:11 2007 +0200
+++ b/src/HOL/Library/SCT_Definition.thy	Wed Jun 13 18:30:15 2007 +0200
@@ -3,7 +3,7 @@
     Author:     Alexander Krauss, TU Muenchen
 *)
 
-header ""
+header ""   (* FIXME proper header *)
 
 theory SCT_Definition
 imports Graphs Infinite_Set
--- a/src/HOL/Library/SCT_Examples.thy	Wed Jun 13 18:30:11 2007 +0200
+++ b/src/HOL/Library/SCT_Examples.thy	Wed Jun 13 18:30:15 2007 +0200
@@ -3,7 +3,7 @@
     Author:     Alexander Krauss, TU Muenchen
 *)
 
-header ""
+header ""   (* FIXME proper header *)
 
 theory SCT_Examples
 imports Size_Change_Termination
--- a/src/HOL/Library/SCT_Implementation.thy	Wed Jun 13 18:30:11 2007 +0200
+++ b/src/HOL/Library/SCT_Implementation.thy	Wed Jun 13 18:30:15 2007 +0200
@@ -3,7 +3,7 @@
     Author:     Alexander Krauss, TU Muenchen
 *)
 
-header ""
+header ""   (* FIXME proper header *)
 
 theory SCT_Implementation
 imports ExecutableSet SCT_Definition
--- a/src/HOL/Library/SCT_Interpretation.thy	Wed Jun 13 18:30:11 2007 +0200
+++ b/src/HOL/Library/SCT_Interpretation.thy	Wed Jun 13 18:30:15 2007 +0200
@@ -3,7 +3,7 @@
     Author:     Alexander Krauss, TU Muenchen
 *)
 
-header ""
+header ""   (* FIXME proper header *)
 
 theory SCT_Interpretation
 imports Main SCT_Misc SCT_Definition
--- a/src/HOL/Library/Size_Change_Termination.thy	Wed Jun 13 18:30:11 2007 +0200
+++ b/src/HOL/Library/Size_Change_Termination.thy	Wed Jun 13 18:30:15 2007 +0200
@@ -3,7 +3,7 @@
     Author:     Alexander Krauss, TU Muenchen
 *)
 
-header ""
+header ""   (* FIXME proper header *)
 
 theory Size_Change_Termination
 imports SCT_Theorem SCT_Interpretation SCT_Implementation