src/HOL/UNITY/LessThan.thy
author wenzelm
Mon, 13 Mar 2000 13:21:39 +0100
changeset 8434 5e4bba59bfaa
parent 7878 43b03d412b82
child 8703 816d8f6513be
permissions -rw-r--r--
use HOLogic.Not; export indexify_names;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     1
(*  Title:      HOL/UNITY/LessThan
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     2
    ID:         $Id$
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     4
    Copyright   1998  University of Cambridge
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     5
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     6
lessThan, greaterThan, atLeast, atMost
5536
130f3d891fb2 tidying and deleting needless parentheses
paulson
parents: 5232
diff changeset
     7
130f3d891fb2 tidying and deleting needless parentheses
paulson
parents: 5232
diff changeset
     8
Could generalize to any linear ordering?
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     9
*)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    10
5232
e5a7cdd07ea5 Tidied; uses records
paulson
parents: 4776
diff changeset
    11
LessThan = Main +
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    12
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    13
constdefs
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    14
7878
43b03d412b82 working version with localTo[C] instead of localTo
paulson
parents: 5536
diff changeset
    15
  (*MOVE TO RELATION.THY??*)
43b03d412b82 working version with localTo[C] instead of localTo
paulson
parents: 5536
diff changeset
    16
  Restrict :: "[ 'a set, ('a*'b) set] => ('a*'b) set"
43b03d412b82 working version with localTo[C] instead of localTo
paulson
parents: 5536
diff changeset
    17
    "Restrict A r == r Int (A Times UNIV)"
43b03d412b82 working version with localTo[C] instead of localTo
paulson
parents: 5536
diff changeset
    18
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    19
  lessThan   :: "nat => nat set"
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    20
     "lessThan n == {i. i<n}"
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    21
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    22
  atMost   :: "nat => nat set"
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    23
     "atMost n == {i. i<=n}"
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    24
 
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    25
  greaterThan   :: "nat => nat set"
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    26
     "greaterThan n == {i. n<i}"
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    27
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    28
  atLeast   :: "nat => nat set"
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    29
     "atLeast n == {i. n<=i}"
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    30
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    31
end