| changeset 30375 | ad2a9dc516ed |
| parent 30331 | 32ccef17d408 |
| child 32139 | e271a64f03ff |
--- a/src/HOL/Library/Lattice_Syntax.thy Sun Mar 08 15:25:28 2009 +0100 +++ b/src/HOL/Library/Lattice_Syntax.thy Sun Mar 08 15:25:29 2009 +0100 @@ -11,7 +11,9 @@ inf (infixl "\<sqinter>" 70) and sup (infixl "\<squnion>" 65) and Inf ("\<Sqinter>_" [900] 900) and - Sup ("\<Squnion>_" [900] 900) + Sup ("\<Squnion>_" [900] 900) and + top ("\<top>") and + bot ("\<bottom>") end (*>*) \ No newline at end of file