src/HOL/Inverse_Image.thy
author wenzelm
Wed, 18 Oct 2000 23:26:42 +0200
changeset 10246 d8c968e6329a
parent 10213 01c2744a3786
child 10832 e33b47e4246d
permissions -rw-r--r--
restart: do not reset theory loader path;

(*  Title:      HOL/Inverse_Image.thy
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1998  University of Cambridge

Inverse image of a function
*)

Inverse_Image = Set +

constdefs
  vimage :: ['a => 'b, 'b set] => ('a set)   (infixr "-``" 90)
    "f-``B  == {x. f(x) : B}"

end