| author | haftmann | 
| Mon, 21 Jun 2010 09:38:20 +0200 | |
| changeset 37475 | 98c6f9dc58d0 | 
| parent 35787 | afdf1c4958b2 | 
| child 41080 | 294956ff285b | 
| permissions | -rw-r--r-- | 
(* Author: Florian Haftmann, TU Muenchen *) header {* Pretty syntax for lattice operations *} theory Lattice_Syntax imports Complete_Lattice begin notation top ("\<top>") and bot ("\<bottom>") and inf (infixl "\<sqinter>" 70) and sup (infixl "\<squnion>" 65) and Inf ("\<Sqinter>_" [900] 900) and Sup ("\<Squnion>_" [900] 900) end