| author | berghofe |
| Fri, 29 Sep 2000 18:02:24 +0200 | |
| changeset 10117 | 8e58b3045e29 |
| parent 10065 | ddb3a014f721 |
| permissions | -rw-r--r-- |
| 7515 | 1 |
(* Title: HOL/Vimage |
2 |
ID: $Id$ |
|
3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
|
4 |
Copyright 1998 University of Cambridge |
|
5 |
||
6 |
Inverse image of a function |
|
7 |
*) |
|
8 |
||
| 4648 | 9 |
Vimage = Set + |
10 |
||
| 10065 | 11 |
constdefs |
12 |
vimage :: ['a => 'b, 'b set] => ('a set) (infixr "-``" 90)
|
|
13 |
"f-``B == {x. f(x) : B}"
|
|
| 4648 | 14 |
|
15 |
end |