src/HOL/UNITY/LessThan.thy
changeset 8948 b797cfa3548d
parent 8947 971aedd340e4
child 8949 d46adac29b71
--- a/src/HOL/UNITY/LessThan.thy	Wed May 24 18:19:04 2000 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,31 +0,0 @@
-(*  Title:      HOL/UNITY/LessThan
-    ID:         $Id$
-    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
-    Copyright   1998  University of Cambridge
-
-lessThan, greaterThan, atLeast, atMost
-
-Could generalize to any linear ordering?
-*)
-
-LessThan = Main +
-
-constdefs
-
-  (*MOVE TO RELATION.THY??*)
-  Restrict :: "[ 'a set, ('a*'b) set] => ('a*'b) set"
-    "Restrict A r == r Int (A <*> UNIV)"
-
-  lessThan   :: "nat => nat set"
-     "lessThan n == {i. i<n}"
-
-  atMost   :: "nat => nat set"
-     "atMost n == {i. i<=n}"
- 
-  greaterThan   :: "nat => nat set"
-     "greaterThan n == {i. n<i}"
-
-  atLeast   :: "nat => nat set"
-     "atLeast n == {i. n<=i}"
-
-end