src/Sequents/LK0.thy
changeset 81125 ec121999a9cb
parent 80924 92d2ceda2370
--- a/src/Sequents/LK0.thy	Sun Oct 06 22:56:07 2024 +0200
+++ b/src/Sequents/LK0.thy	Tue Oct 08 12:10:35 2024 +0200
@@ -24,7 +24,7 @@
   True         :: o
   False        :: o
   equal        :: "['a,'a] \<Rightarrow> o"     (infixl \<open>=\<close> 50)
-  Not          :: "o \<Rightarrow> o"           (\<open>\<not> _\<close> [40] 40)
+  Not          :: "o \<Rightarrow> o"           (\<open>(\<open>open_block notation=\<open>prefix \<not>\<close>\<close>\<not> _)\<close> [40] 40)
   conj         :: "[o,o] \<Rightarrow> o"       (infixr \<open>\<and>\<close> 35)
   disj         :: "[o,o] \<Rightarrow> o"       (infixr \<open>\<or>\<close> 30)
   imp          :: "[o,o] \<Rightarrow> o"       (infixr \<open>\<longrightarrow>\<close> 25)