Closures.thy
changeset 241 68d48522ea9a
parent 240 17aa8c8fbe7d
child 252 8e2c497d699e
--- a/Closures.thy	Mon Sep 05 15:42:29 2011 +0000
+++ b/Closures.thy	Mon Sep 05 20:59:50 2011 +0000
@@ -209,7 +209,7 @@
 qed
 
 
-subsection {* Non-regularity for languages *}
+subsection {* Continuation lemma for showing non-regularity of languages *}
 
 lemma continuation_lemma:
   fixes A B::"'a::finite lang"
@@ -243,7 +243,7 @@
 qed
 
 
-subsubsection {* The language @{text "a ^ n b ^ n"} is not regular *}
+subsection {* The language @{text "a\<^sup>n b\<^sup>n"} is not regular *}
 
 abbreviation
   replicate_rev ("_ ^^^ _" [100, 100] 100)