src/HOL/Library/SCT_Definition.thy
changeset 22665 cf152ff55d16
parent 22371 c9f5895972b0
child 22744 5cbe966d67a2
--- a/src/HOL/Library/SCT_Definition.thy	Fri Apr 13 21:26:34 2007 +0200
+++ b/src/HOL/Library/SCT_Definition.thy	Fri Apr 13 21:26:35 2007 +0200
@@ -3,14 +3,16 @@
     Author:     Alexander Krauss, TU Muenchen
 *)
 
+header ""
+
 theory SCT_Definition
 imports Graphs Infinite_Set
 begin
 
-section {* Size-Change Graphs *}
+subsection {* Size-Change Graphs *}
 
 datatype sedge =
-  LESS ("\<down>")
+    LESS ("\<down>")
   | LEQ ("\<Down>")
 
 instance sedge :: times ..
@@ -42,7 +44,7 @@
 types acg = "(nat, scg) graph"
 
 
-section {* Size-Change Termination *}
+subsection {* Size-Change Termination *}
 
 abbreviation (input)
   "desc P Q == ((\<exists>n.\<forall>i\<ge>n. P i) \<and> (\<exists>\<^sub>\<infinity>i. Q i))"
@@ -97,5 +99,4 @@
 where
   "SCT' A = no_bad_graphs (tcl A)"
 
-
-end
\ No newline at end of file
+end