src/HOL/Inverse_Image.thy
author wenzelm
Fri, 03 Nov 2000 21:27:06 +0100
changeset 10379 93630e0c5ae9
parent 10213 01c2744a3786
child 10832 e33b47e4246d
permissions -rw-r--r--
improved handling of "that": insert into goal, only declare as Pure "intro"; eliminated functor;

(*  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