src/HOL/Inverse_Image.thy
author paulson
Tue, 19 Dec 2000 15:20:23 +0100
changeset 10706 f02834001fca
parent 10213 01c2744a3786
child 10832 e33b47e4246d
permissions -rw-r--r--
re-orienting equations with 0, 1, 2 on the lhs

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