diff -r e965391e2864 -r cf152ff55d16 src/HOL/Library/ExecutableSet.thy --- a/src/HOL/Library/ExecutableSet.thy Fri Apr 13 21:26:34 2007 +0200 +++ b/src/HOL/Library/ExecutableSet.thy Fri Apr 13 21:26:35 2007 +0200 @@ -9,7 +9,7 @@ imports Main begin -section {* Definitional rewrites *} +subsection {* Definitional rewrites *} instance set :: (eq) eq .. @@ -40,9 +40,9 @@ lemmas [symmetric, code inline] = filter_set_def -section {* Operations on lists *} +subsection {* Operations on lists *} -subsection {* Basic definitions *} +subsubsection {* Basic definitions *} definition flip :: "('a \ 'b \ 'c) \ 'b \ 'a \ 'c" where @@ -107,7 +107,7 @@ by (induct xs) simp_all -subsection {* Derived definitions *} +subsubsection {* Derived definitions *} function unionl :: "'a list \ 'a list \ 'a list" where @@ -169,7 +169,7 @@ "map_inter xs f = intersects (map f xs)" -section {* Isomorphism proofs *} +subsection {* Isomorphism proofs *} lemma iso_member: "member xs x \ x \ set xs" @@ -248,7 +248,7 @@ "set (filter P xs) = filter_set P (set xs)" unfolding filter_set_def by (induct xs) auto -section {* code generator setup *} +subsection {* code generator setup *} ML {* nonfix inter; @@ -317,7 +317,7 @@ filter_set \ filter -subsection {* type serializations *} +subsubsection {* type serializations *} types_code set ("_ list") @@ -333,7 +333,7 @@ *} -subsection {* const serializations *} +subsubsection {* const serializations *} consts_code "{}" ("[]")