diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Induct/PropLog.thy --- a/src/HOL/Induct/PropLog.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Induct/PropLog.thy Fri Sep 20 19:51:08 2024 +0200 @@ -22,13 +22,13 @@ datatype 'a pl = false - | var 'a ("#_" [1000]) - | imp "'a pl" "'a pl" (infixr "\" 90) + | var 'a (\#_\ [1000]) + | imp "'a pl" "'a pl" (infixr \\\ 90) subsection \The proof system\ -inductive thms :: "['a pl set, 'a pl] \ bool" (infixl "\" 50) +inductive thms :: "['a pl set, 'a pl] \ bool" (infixl \\\ 50) for H :: "'a pl set" where H: "p \ H \ H \ p" @@ -42,7 +42,7 @@ subsubsection \Semantics of propositional logic.\ -primrec eval :: "['a set, 'a pl] => bool" ("_[[_]]" [100,0] 100) +primrec eval :: "['a set, 'a pl] => bool" (\_[[_]]\ [100,0] 100) where "tt[[false]] = False" | "tt[[#v]] = (v \ tt)" @@ -67,7 +67,7 @@ is \p\. \ -definition sat :: "['a pl set, 'a pl] => bool" (infixl "\" 50) +definition sat :: "['a pl set, 'a pl] => bool" (infixl \\\ 50) where "H \ p = (\tt. (\q\H. tt[[q]]) \ tt[[p]])"