src/ZF/Perm.thy
changeset 16417 9bc16273c2d4
parent 14883 ca000a495448
child 24893 b8ef7afe3a6b
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     9   -- Lemmas for the Schroeder-Bernstein Theorem
     9   -- Lemmas for the Schroeder-Bernstein Theorem
    10 *)
    10 *)
    11 
    11 
    12 header{*Injections, Surjections, Bijections, Composition*}
    12 header{*Injections, Surjections, Bijections, Composition*}
    13 
    13 
    14 theory Perm = func:
    14 theory Perm imports func begin
    15 
    15 
    16 constdefs
    16 constdefs
    17 
    17 
    18   (*composition of relations and functions; NOT Suppes's relative product*)
    18   (*composition of relations and functions; NOT Suppes's relative product*)
    19   comp     :: "[i,i]=>i"      (infixr "O" 60)
    19   comp     :: "[i,i]=>i"      (infixr "O" 60)