| author | bulwahn | 
| Tue, 02 Mar 2010 22:13:32 +0100 | |
| changeset 35536 | 1f980bbc6ad8 | 
| parent 32139 | e271a64f03ff | 
| child 35787 | afdf1c4958b2 | 
| permissions | -rw-r--r-- | 
| 30330 | 1 | (* Author: Florian Haftmann, TU Muenchen *) | 
| 2 | ||
| 3 | header {* Pretty syntax for lattice operations *}
 | |
| 4 | ||
| 30331 | 5 | (*<*) | 
| 30330 | 6 | theory Lattice_Syntax | 
| 32139 | 7 | imports Complete_Lattice | 
| 30330 | 8 | begin | 
| 9 | ||
| 10 | notation | |
| 32139 | 11 |   top ("\<top>") and
 | 
| 12 |   bot ("\<bottom>") and
 | |
| 30330 | 13 | inf (infixl "\<sqinter>" 70) and | 
| 14 | sup (infixl "\<squnion>" 65) and | |
| 15 |   Inf  ("\<Sqinter>_" [900] 900) and
 | |
| 32139 | 16 |   Sup  ("\<Squnion>_" [900] 900)
 | 
| 30330 | 17 | |
| 30331 | 18 | end | 
| 19 | (*>*) |