src/HOL/Relation.thy
changeset 3439 54785105178c
parent 1983 f3f7bf0079fa
child 3499 ce1664057431
equal deleted inserted replaced
3438:8d63ff01d37e 3439:54785105178c
     7 Relation = Prod +
     7 Relation = Prod +
     8 consts
     8 consts
     9     id          :: "('a * 'a)set"               (*the identity relation*)
     9     id          :: "('a * 'a)set"               (*the identity relation*)
    10     O           :: "[('b * 'c)set, ('a * 'b)set] => ('a * 'c)set" (infixr 60)
    10     O           :: "[('b * 'c)set, ('a * 'b)set] => ('a * 'c)set" (infixr 60)
    11     trans       :: "('a * 'a)set => bool"       (*transitivity predicate*)
    11     trans       :: "('a * 'a)set => bool"       (*transitivity predicate*)
    12     converse    :: "('a*'b) set => ('b*'a) set"
    12     inverse    :: "('a*'b) set => ('b*'a) set"     ("(_^-1)" [1000] 1000)
    13     "^^"        :: "[('a*'b) set,'a set] => 'b set" (infixl 90)
    13     "^^"        :: "[('a*'b) set,'a set] => 'b set" (infixl 90)
    14     Domain      :: "('a*'b) set => 'a set"
    14     Domain      :: "('a*'b) set => 'a set"
    15     Range       :: "('a*'b) set => 'b set"
    15     Range       :: "('a*'b) set => 'b set"
    16 defs
    16 defs
    17     id_def        "id == {p. ? x. p = (x,x)}"
    17     id_def        "id == {p. ? x. p = (x,x)}"
    18     comp_def      "r O s == {(x,z). ? y. (x,y):s & (y,z):r}"
    18     comp_def      "r O s == {(x,z). ? y. (x,y):s & (y,z):r}"
    19     trans_def     "trans(r) == (!x y z. (x,y):r --> (y,z):r --> (x,z):r)"
    19     trans_def     "trans(r) == (!x y z. (x,y):r --> (y,z):r --> (x,z):r)"
    20     converse_def  "converse(r) == {(y,x). (x,y):r}"
    20     inverse_def   "r^-1 == {(y,x). (x,y):r}"
    21     Domain_def    "Domain(r) == {x. ? y. (x,y):r}"
    21     Domain_def    "Domain(r) == {x. ? y. (x,y):r}"
    22     Range_def     "Range(r) == Domain(converse(r))"
    22     Range_def     "Range(r) == Domain(r^-1)"
    23     Image_def     "r ^^ s == {y. ? x:s. (x,y):r}"
    23     Image_def     "r ^^ s == {y. ? x:s. (x,y):r}"
    24 end
    24 end