src/HOL/IMP/Collecting1.thy
changeset 68778 4566bac4517d
parent 67613 ce654b0e6d69
child 69597 ff784d5a5bfb
--- a/src/HOL/IMP/Collecting1.thy	Mon Aug 20 20:54:40 2018 +0200
+++ b/src/HOL/IMP/Collecting1.thy	Tue Aug 21 17:29:46 2018 +0200
@@ -1,9 +1,9 @@
+subsection "A small step semantics on annotated commands"
+
 theory Collecting1
 imports Collecting
 begin
 
-subsection "A small step semantics on annotated commands"
-
 text\<open>The idea: the state is propagated through the annotated command as an
 annotation @{term "{s}"}, all other annotations are @{term "{}"}. It is easy
 to show that this semantics approximates the collecting semantics.\<close>