src/HOL/Integ/Relation.thy
author paulson
Thu, 15 Jul 1999 10:34:37 +0200
changeset 7010 63120b6dca50
parent 972 e61b058d58d2
permissions -rw-r--r--
more renaming of theorems from _nat to _int (corresponding to a function that was similarly renamed some time ago Also new theorem zmult_int

(*  Title: 	Relation.thy
    ID:         $Id$
    Author: 	Riccardo Mattolini, Dip. Sistemi e Informatica
        and	Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1994 Universita' di Firenze
    Copyright   1993  University of Cambridge

Functions represented as relations in Higher-Order Set Theory 
*)

Relation = Trancl +
consts
    converse    ::      "('a*'a) set => ('a*'a) set"
    "^^"        ::      "[('a*'a) set,'a set] => 'a set" (infixl 90)
    Domain      ::      "('a*'a) set => 'a set"
    Range       ::      "('a*'a) set => 'a set"

defs
    converse_def  "converse(r) == {z. (? w:r. ? x y. w=(x,y) & z=(y,x))}"
    Domain_def    "Domain(r) == {z. ! x. (z=x --> (? y. (x,y):r))}"
    Range_def     "Range(r) == Domain(converse(r))"
    Image_def     "r ^^ s == {y. y:Range(r) &  (? x:s. (x,y):r)}"

end