src/HOL/Library/LaTeXsugar.thy
changeset 16110 c423bb89186d
parent 15690 1da2cfd1ca45
child 19674 22b635240905
--- a/src/HOL/Library/LaTeXsugar.thy	Sun May 29 12:41:40 2005 +0200
+++ b/src/HOL/Library/LaTeXsugar.thy	Mon May 30 08:21:58 2005 +0200
@@ -20,6 +20,12 @@
   "_case_syntax":: "['a, cases_syn] => 'b"
   ("(\<^raw:\textsf{>case\<^raw:}> _ \<^raw:\textsf{>of\<^raw:}>/ _)" 10)
 
+(* should become standard syntax once x-symbols supports it *)
+syntax (latex)
+  nexists :: "('a => bool) => bool"           (binder "\<nexists>" 10)
+translations
+  "\<nexists>x. P" <= "\<not>(\<exists>x. P)"
+
 (* SETS *)
 
 (* empty set *)