src/HOL/ex/set.thy
changeset 19982 e4d50f8f3722
parent 18391 2e901da7cd3a
child 24573 5bbdc9b60648
equal deleted inserted replaced
19981:c0f124a0d385 19982:e4d50f8f3722
     2     ID:         $Id$
     2     ID:         $Id$
     3     Author:     Tobias Nipkow and Lawrence C Paulson
     3     Author:     Tobias Nipkow and Lawrence C Paulson
     4     Copyright   1991  University of Cambridge
     4     Copyright   1991  University of Cambridge
     5 *)
     5 *)
     6 
     6 
     7 header {* Set Theory examples: Cantor's Theorem, Schröder-Berstein Theorem, etc. *}
     7 header {* Set Theory examples: Cantor's Theorem, Schröder-Bernstein Theorem, etc. *}
     8 
     8 
     9 theory set imports Main begin
     9 theory set imports Main begin
    10 
    10 
    11 text{*
    11 text{*
    12   These two are cited in Benzmueller and Kohlhase's system description
    12   These two are cited in Benzmueller and Kohlhase's system description