src/HOL/Fun.thy
author nipkow
Fri, 04 Apr 1997 16:33:28 +0200
changeset 2912 3fac3e8d5d3e
parent 1475 7f5a4cd08209
child 4059 59c1422c9da5
permissions -rw-r--r--
moved inj and surj from Set to Fun and Inv -> inv.

(*  Title:      HOL/Fun.thy
    ID:         $Id$
    Author:     Tobias Nipkow, Cambridge University Computer Laboratory
    Copyright   1994  University of Cambridge

Notions about functions.
*)

Fun = Set +

consts

  inj, surj     :: ('a => 'b) => bool                   (*inj/surjective*)
  inj_onto      :: ['a => 'b, 'a set] => bool
  inv           :: ('a => 'b) => ('b => 'a)

defs

  inj_def       "inj f          == ! x y. f(x)=f(y) --> x=y"
  inj_onto_def  "inj_onto f A   == ! x:A. ! y:A. f(x)=f(y) --> x=y"
  surj_def      "surj f         == ! y. ? x. y=f(x)"
  inv_def       "inv(f::'a=>'b) == (% y. @x. f(x)=y)"

end