Ord.ML
author clasohm
Thu, 08 Dec 1994 12:50:38 +0100
changeset 199 ad45e477926c
parent 171 16c4ea954511
permissions -rw-r--r--
replaced store_thm by bind_thm
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
118
5b96b1252cdc HOL/Ord.thy,.ML: files now have header comments
lcp
parents: 0
diff changeset
     1
(*  Title: 	HOL/Ord.ML
5b96b1252cdc HOL/Ord.thy,.ML: files now have header comments
lcp
parents: 0
diff changeset
     2
    ID:         $Id$
5b96b1252cdc HOL/Ord.thy,.ML: files now have header comments
lcp
parents: 0
diff changeset
     3
    Author: 	Tobias Nipkow, Cambridge University Computer Laboratory
5b96b1252cdc HOL/Ord.thy,.ML: files now have header comments
lcp
parents: 0
diff changeset
     4
    Copyright   1993  University of Cambridge
5b96b1252cdc HOL/Ord.thy,.ML: files now have header comments
lcp
parents: 0
diff changeset
     5
5b96b1252cdc HOL/Ord.thy,.ML: files now have header comments
lcp
parents: 0
diff changeset
     6
The type class for ordered types
5b96b1252cdc HOL/Ord.thy,.ML: files now have header comments
lcp
parents: 0
diff changeset
     7
*)
5b96b1252cdc HOL/Ord.thy,.ML: files now have header comments
lcp
parents: 0
diff changeset
     8
0
7949f97df77a Initial revision
clasohm
parents:
diff changeset
     9
open Ord;
7949f97df77a Initial revision
clasohm
parents:
diff changeset
    10
7949f97df77a Initial revision
clasohm
parents:
diff changeset
    11
val [prem] = goalw Ord.thy [mono_def]
7949f97df77a Initial revision
clasohm
parents:
diff changeset
    12
    "[| !!A B. A <= B ==> f(A) <= f(B) |] ==> mono(f)";
7949f97df77a Initial revision
clasohm
parents:
diff changeset
    13
by (REPEAT (ares_tac [allI, impI, prem] 1));
171
16c4ea954511 replaced 'val ... = result()' by 'qed "..."'
clasohm
parents: 118
diff changeset
    14
qed "monoI";
0
7949f97df77a Initial revision
clasohm
parents:
diff changeset
    15
7949f97df77a Initial revision
clasohm
parents:
diff changeset
    16
val [major,minor] = goalw Ord.thy [mono_def]
7949f97df77a Initial revision
clasohm
parents:
diff changeset
    17
    "[| mono(f);  A <= B |] ==> f(A) <= f(B)";
7949f97df77a Initial revision
clasohm
parents:
diff changeset
    18
by (rtac (major RS spec RS spec RS mp) 1);
7949f97df77a Initial revision
clasohm
parents:
diff changeset
    19
by (rtac minor 1);
171
16c4ea954511 replaced 'val ... = result()' by 'qed "..."'
clasohm
parents: 118
diff changeset
    20
qed "monoD";
0
7949f97df77a Initial revision
clasohm
parents:
diff changeset
    21