diff -r a730a5a0bab9 -r 89e6605c4ca4 thys/Positions.thy --- a/thys/Positions.thy Tue Jul 23 21:21:49 2019 +0100 +++ b/thys/Positions.thy Mon Jul 29 09:37:20 2019 +0100 @@ -3,9 +3,9 @@ imports "Spec" "Lexer" begin -chapter {* An alternative definition for POSIX values *} +chapter \An alternative definition for POSIX values\ -section {* Positions in Values *} +section \Positions in Values\ fun at :: "val \ nat list \ val" @@ -76,7 +76,7 @@ -section {* Orderings *} +section \Orderings\ definition prefix_list:: "'a list \ 'a list \ bool" ("_ \pre _" [60,59] 60) @@ -128,7 +128,7 @@ -section {* POSIX Ordering of Values According to Okui \& Suzuki *} +section \POSIX Ordering of Values According to Okui \& Suzuki\ definition PosOrd:: "val \ nat list \ val \ bool" ("_ \val _ _" [60, 60, 59] 60) @@ -512,7 +512,7 @@ -section {* The Posix Value is smaller than any other Value *} +section \The Posix Value is smaller than any other Value\ lemma Posix_PosOrd: