src/HOL/Vimage.thy
author berghofe
Fri, 24 Jul 1998 13:19:38 +0200
changeset 5184 9b8547a9496a
parent 4648 f04da668581c
child 7515 0c05469cad57
permissions -rw-r--r--
Adapted to new datatype package.
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
4648
f04da668581c New theory of the inverse image of a function
paulson
parents:
diff changeset
     1
Vimage = Set +
f04da668581c New theory of the inverse image of a function
paulson
parents:
diff changeset
     2
f04da668581c New theory of the inverse image of a function
paulson
parents:
diff changeset
     3
consts
f04da668581c New theory of the inverse image of a function
paulson
parents:
diff changeset
     4
  "-``"          :: ['a => 'b, 'b set] => ('a set)   (infixr 90)
f04da668581c New theory of the inverse image of a function
paulson
parents:
diff changeset
     5
f04da668581c New theory of the inverse image of a function
paulson
parents:
diff changeset
     6
defs
f04da668581c New theory of the inverse image of a function
paulson
parents:
diff changeset
     7
  vimage_def     "f-``B           == {x. f(x) : B}"
f04da668581c New theory of the inverse image of a function
paulson
parents:
diff changeset
     8
f04da668581c New theory of the inverse image of a function
paulson
parents:
diff changeset
     9
end