8924
|
1 |
(* Title: HOL/SetInterval.thy
|
|
2 |
ID: $Id$
|
|
3 |
Author: Tobias Nipkow
|
8957
|
4 |
Copyright 2000 TU Muenchen
|
8924
|
5 |
|
|
6 |
lessThan, greaterThan, atLeast, atMost
|
|
7 |
*)
|
|
8 |
|
10214
|
9 |
SetInterval = equalities + NatArith +
|
8924
|
10 |
|
|
11 |
constdefs
|
|
12 |
lessThan :: "('a::ord) => 'a set" ("(1{.._'(})")
|
|
13 |
"{..u(} == {x. x<u}"
|
|
14 |
|
|
15 |
atMost :: "('a::ord) => 'a set" ("(1{.._})")
|
|
16 |
"{..u} == {x. x<=u}"
|
|
17 |
|
|
18 |
greaterThan :: "('a::ord) => 'a set" ("(1{')_..})")
|
|
19 |
"{)l..} == {x. l<x}"
|
|
20 |
|
|
21 |
atLeast :: "('a::ord) => 'a set" ("(1{_..})")
|
|
22 |
"{l..} == {x. l<=x}"
|
|
23 |
|
|
24 |
end
|