src/HOL/Library/LaTeXsugar.thy
changeset 27688 397de75836a1
parent 27487 c8a6ce181805
child 29493 ddcbd5e4041d
--- a/src/HOL/Library/LaTeXsugar.thy	Sun Jul 27 20:08:16 2008 +0200
+++ b/src/HOL/Library/LaTeXsugar.thy	Mon Jul 28 20:49:07 2008 +0200
@@ -30,17 +30,15 @@
 (* SETS *)
 
 (* empty set *)
-syntax (latex output)
-  "_emptyset" :: "'a set"              ("\<emptyset>")
-translations
-  "_emptyset"      <= "{}"
+notation (latex)
+  "{}" ("\<emptyset>")
 
 (* insert *)
 translations 
   "{x} \<union> A" <= "insert x A"
   "{x,y}" <= "{x} \<union> {y}"
   "{x,y} \<union> A" <= "{x} \<union> ({y} \<union> A)"
-  "{x}" <= "{x} \<union> _emptyset"
+  "{x}" <= "{x} \<union> \<emptyset>"
 
 (* set comprehension *)
 syntax (latex output)