src/HOL/IMP/Fold.thy
changeset 44850 a6095c96a89b
parent 44070 cebb7abb54b1
child 44890 22f665a2e91c
--- a/src/HOL/IMP/Fold.thy	Tue Sep 06 14:25:16 2011 +0200
+++ b/src/HOL/IMP/Fold.thy	Fri Sep 09 06:45:39 2011 +0200
@@ -2,7 +2,7 @@
 
 theory Fold imports Sem_Equiv begin
 
-section "Simple folding of arithmetic expressions"
+subsection "Simple folding of arithmetic expressions"
 
 types
   tab = "name \<Rightarrow> val option"
@@ -226,7 +226,7 @@
 
 
 
-section {* More ambitious folding including boolean expressions *}
+subsection {* More ambitious folding including boolean expressions *}
 
 
 fun bsimp_const :: "bexp \<Rightarrow> tab \<Rightarrow> bexp" where