src/FOL/IFOL.thy
changeset 80923 6c9628a116cc
parent 80917 2a77bc3b4eac
child 81011 6d34c2bedaa3
--- a/src/FOL/IFOL.thy	Sun Sep 22 16:04:44 2024 +0200
+++ b/src/FOL/IFOL.thy	Sun Sep 22 16:12:15 2024 +0200
@@ -32,7 +32,7 @@
 typedecl o
 
 judgment
-  Trueprop :: \<open>o \<Rightarrow> prop\<close>  (\<open>(_)\<close> 5)
+  Trueprop :: \<open>o \<Rightarrow> prop\<close>  (\<open>(\<open>notation=judgment\<close>_)\<close> 5)
 
 
 subsubsection \<open>Equality\<close>