Ord.thy
author wenzelm
Mon, 04 Oct 1993 15:43:54 +0100
changeset 4 d199410f1db1
parent 0 7949f97df77a
child 118 5b96b1252cdc
permissions -rw-r--r--
HOL/hol.thy renamed mk_alt_ast_tr' to alt_ast_tr'; added alternative quantifier THE; replaced Ast by Syntax; HOL/set.thy replaced HOL.mk_alt_ast_tr' by HOL.alt_ast_tr';

Ord = HOL +
classes
  ord < term
consts
  "<", "<="     :: "['a::ord, 'a] => bool"              (infixl 50)
  mono		:: "['a::ord => 'b::ord] => bool"       (*monotonicity*)
  min,max	:: "['a::ord,'a] => 'a"

rules

mono_def  "mono(f)  == (!A B. A <= B --> f(A) <= f(B))"
min_def   "min(a,b) == if(a <= b, a, b)"
max_def   "max(a,b) == if(a <= b, b, a)"

end