src/HOL/Lattice/Lattice.thy
changeset 35317 d57da4abb47d
parent 25469 f81b3be9dfdd
child 37678 0040bafffdef
equal deleted inserted replaced
35316:870dfea4f9c0 35317:d57da4abb47d
     1 (*  Title:      HOL/Lattice/Lattice.thy
     1 (*  Title:      HOL/Lattice/Lattice.thy
     2     ID:         $Id$
       
     3     Author:     Markus Wenzel, TU Muenchen
     2     Author:     Markus Wenzel, TU Muenchen
     4 *)
     3 *)
     5 
     4 
     6 header {* Lattices *}
     5 header {* Lattices *}
     7 
     6 
    13   A \emph{lattice} is a partial order with infimum and supremum of any
    12   A \emph{lattice} is a partial order with infimum and supremum of any
    14   two elements (thus any \emph{finite} number of elements have bounds
    13   two elements (thus any \emph{finite} number of elements have bounds
    15   as well).
    14   as well).
    16 *}
    15 *}
    17 
    16 
    18 axclass lattice \<subseteq> partial_order
    17 class lattice =
    19   ex_inf: "\<exists>inf. is_inf x y inf"
    18   assumes ex_inf: "\<exists>inf. is_inf x y inf"
    20   ex_sup: "\<exists>sup. is_sup x y sup"
    19   assumes ex_sup: "\<exists>sup. is_sup x y sup"
    21 
    20 
    22 text {*
    21 text {*
    23   The @{text \<sqinter>} (meet) and @{text \<squnion>} (join) operations select such
    22   The @{text \<sqinter>} (meet) and @{text \<squnion>} (join) operations select such
    24   infimum and supremum elements.
    23   infimum and supremum elements.
    25 *}
    24 *}