fixed bugs
authornipkow
Thu, 27 Jan 2005 13:33:21 +0100
changeset 15476 b8cb20cc0c0b
parent 15475 fdf9434b04ea
child 15477 5058984779b9
fixed bugs
src/HOL/Library/LaTeXsugar.thy
src/HOL/Library/OptionalSugar.thy
--- a/src/HOL/Library/LaTeXsugar.thy	Thu Jan 27 12:37:02 2005 +0100
+++ b/src/HOL/Library/LaTeXsugar.thy	Thu Jan 27 13:33:21 2005 +0100
@@ -32,6 +32,7 @@
 translations 
   "{x} \<union> A" <= "insert x A"
   "{x,y} \<union> A" <= "{x} \<union> ({y} \<union> A)"
+  "{x}" <= "{x} \<union> _emptyset"
 
 (* set comprehension *)
 syntax (latex output)
--- a/src/HOL/Library/OptionalSugar.thy	Thu Jan 27 12:37:02 2005 +0100
+++ b/src/HOL/Library/OptionalSugar.thy	Thu Jan 27 13:33:21 2005 +0100
@@ -3,7 +3,7 @@
     Author:     Gerwin Klain, Tobias Nipkow
     Copyright   2005 NICTA and TUM
 *)
-
+(*<*)
 theory OptionalSugar
 imports LaTeXsugar
 begin
@@ -34,4 +34,5 @@
   "_bind (DUMMY#p) e" <= "_bind p (tl e)"
 
 
-end
\ No newline at end of file
+end
+(*>*)