Ord.ML
author lcp
Fri, 11 Nov 1994 10:35:03 +0100
changeset 170 3a8d722fd3ff
parent 118 5b96b1252cdc
child 171 16c4ea954511
permissions -rw-r--r--
HOL,ZF/Makefile: enclosed multiple "use" calls in parentheses. This ensures that if one dies, all die. BUT NOT Pure/Makefile, where PolyML.use"POLY" makes the identifier "use" visible.

(*  Title: 	HOL/Ord.ML
    ID:         $Id$
    Author: 	Tobias Nipkow, Cambridge University Computer Laboratory
    Copyright   1993  University of Cambridge

The type class for ordered types
*)

open Ord;

val [prem] = goalw Ord.thy [mono_def]
    "[| !!A B. A <= B ==> f(A) <= f(B) |] ==> mono(f)";
by (REPEAT (ares_tac [allI, impI, prem] 1));
val monoI = result();

val [major,minor] = goalw Ord.thy [mono_def]
    "[| mono(f);  A <= B |] ==> f(A) <= f(B)";
by (rtac (major RS spec RS spec RS mp) 1);
by (rtac minor 1);
val monoD = result();