src/HOL/AxClasses/Lattice/LatInsts.thy
author wenzelm
Tue, 27 May 1997 15:45:07 +0200
changeset 3362 0b268cff9344
parent 2606 27cdd600a3b1
permissions -rw-r--r--
NJ 1.09.2x as factory default!

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

Some lattice instantiations.
*)

LatInsts = LatPreInsts +


(* linear orders are lattices *)

instance
  linear_order < lattice                (allI, exI, min_is_inf, max_is_sup)


(* complete lattices are lattices *)

instance
  clattice < lattice                    (allI, exI, Inf_is_inf, Sup_is_sup)


(* products of lattices are lattices *)

instance
  "*" :: (lattice, lattice) lattice     (allI, exI, prod_is_inf, prod_is_sup)

instance
  fun :: (term, lattice) lattice        (allI, exI, fun_is_inf, fun_is_sup)


(* duals of lattices are lattices *)

instance
  dual :: (lattice) lattice             (allI, exI, dual_is_inf, dual_is_sup)

(*FIXME bug workaround (see also OrdInsts.thy)*)
instance
  dual :: (linear_order) linear_order   (le_dual_linear)

end