diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Hoare/Separation.thy --- a/src/HOL/Hoare/Separation.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Hoare/Separation.thy Fri Sep 20 19:51:08 2024 +0200 @@ -19,7 +19,7 @@ text\The semantic definition of a few connectives:\ -definition ortho :: "heap \ heap \ bool" (infix "\" 55) +definition ortho :: "heap \ heap \ bool" (infix \\\ 55) where "h1 \ h2 \ dom h1 \ dom h2 = {}" definition is_empty :: "heap \ bool" @@ -51,10 +51,10 @@ bound Hs - otherwise they may bind the implicit H.\ syntax - "_emp" :: "bool" ("emp") - "_singl" :: "nat \ nat \ bool" ("[_ \ _]") - "_star" :: "bool \ bool \ bool" (infixl "**" 60) - "_wand" :: "bool \ bool \ bool" (infixl "-*" 60) + "_emp" :: "bool" (\emp\) + "_singl" :: "nat \ nat \ bool" (\[_ \ _]\) + "_star" :: "bool \ bool \ bool" (infixl \**\ 60) + "_wand" :: "bool \ bool \ bool" (infixl \-*\ 60) (* FIXME does not handle "_idtdummy" *) ML \