src/HOL/AxClasses/Lattice/Lattice.thy
author clasohm
Wed, 20 Mar 1996 13:21:12 +0100
changeset 1589 fd6a571cb2b0
parent 1440 de6f18da81bb
child 2606 27cdd600a3b1
permissions -rw-r--r--
added warning and automatic deactivation of HTML generation if we cannot write .theory_list.txt; fixed bug which occured when index_path's value is "/"

(*  Title:      Lattice.thy
    ID:         $Id$
    Author:     Markus Wenzel, TU Muenchen

Lattices are orders with binary (finitary) infima and suprema.
*)

Lattice = Order +

axclass
  lattice < order
  ex_inf       "ALL x y. EX inf. is_inf x y inf"
  ex_sup       "ALL x y. EX sup. is_sup x y sup"

consts
  "&&"          :: "['a::lattice, 'a] => 'a"       (infixl 70)
  "||"          :: "['a::lattice, 'a] => 'a"       (infixl 65)

defs
  inf_def       "x && y == @inf. is_inf x y inf"
  sup_def       "x || y == @sup. is_sup x y sup"

end