src/ZF/equalities.thy
changeset 58871 c399ae4b836f
parent 58860 fee7cfa69c50
child 60770 240563fbf41d
equal deleted inserted replaced
58870:e2c0d8ef29cb 58871:c399ae4b836f
     1 (*  Title:      ZF/equalities.thy
     1 (*  Title:      ZF/equalities.thy
     2     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     2     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     3     Copyright   1992  University of Cambridge
     3     Copyright   1992  University of Cambridge
     4 *)
     4 *)
     5 
     5 
     6 header{*Basic Equalities and Inclusions*}
     6 section{*Basic Equalities and Inclusions*}
     7 
     7 
     8 theory equalities imports pair begin
     8 theory equalities imports pair begin
     9 
     9 
    10 text{*These cover union, intersection, converse, domain, range, etc.  Philippe
    10 text{*These cover union, intersection, converse, domain, range, etc.  Philippe
    11 de Groote proved many of the inclusions.*}
    11 de Groote proved many of the inclusions.*}