src/HOL/Set.thy
changeset 15140 322485b816ac
parent 15131 c69542757a4d
child 15206 09d78ec709c7
equal deleted inserted replaced
15139:58cd3404cf75 15140:322485b816ac
     4 *)
     4 *)
     5 
     5 
     6 header {* Set theory for higher-order logic *}
     6 header {* Set theory for higher-order logic *}
     7 
     7 
     8 theory Set
     8 theory Set
     9 import HOL
     9 imports HOL
    10 begin
    10 begin
    11 
    11 
    12 text {* A set in HOL is simply a predicate. *}
    12 text {* A set in HOL is simply a predicate. *}
    13 
    13 
    14 
    14