1
Vimage = Set +
2
3
consts
4
"-``" :: ['a => 'b, 'b set] => ('a set) (infixr 90)
5
6
defs
7
vimage_def "f-``B == {x. f(x) : B}"
8
9
end