src/HOL/AxClasses/Lattice/LatMorph.thy
author paulson
Tue, 16 Jul 1996 15:49:46 +0200
changeset 1868 836950047d85
parent 1573 6d66b59f94a9
permissions -rw-r--r--
Put in minimal simpset to avoid excessive simplification, just as in revision 1.9 of HOL/indrule.ML

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

Some lattice morphisms.

TODO:
  more morphisms (?)
  more theorems
*)

LatMorph = LatInsts +

constdefs
  is_mono       :: "('a::le => 'b::le) => bool"
  "is_mono f == ALL x y. x [= y --> f x [= f y"

  is_inf_morph  :: "('a::lattice => 'b::lattice) => bool"
  "is_inf_morph f == ALL x y. f (x && y) = f x && f y"

  is_sup_morph  :: "('a::lattice => 'b::lattice) => bool"
  "is_sup_morph f == ALL x y. f (x || y) = f x || f y"

  is_Inf_morph  :: "('a::clattice => 'b::clattice) => bool"
  "is_Inf_morph f == ALL A. f (Inf A) = Inf {f x |x. x:A}"

  is_Sup_morph  :: "('a::clattice => 'b::clattice) => bool"
  "is_Sup_morph f == ALL A. f (Sup A) = Sup {f x |x. x:A}"

end