src/ZF/upair.thy
changeset 65449 c82e63b11b8b
parent 63901 4ce989e962e0
child 68233 5e0e9376b2b0
equal deleted inserted replaced
65448:9bc3b57c1fa7 65449:c82e63b11b8b
    10 *)
    10 *)
    11 
    11 
    12 section\<open>Unordered Pairs\<close>
    12 section\<open>Unordered Pairs\<close>
    13 
    13 
    14 theory upair
    14 theory upair
    15 imports ZF
    15 imports ZF_Base
    16 keywords "print_tcset" :: diag
    16 keywords "print_tcset" :: diag
    17 begin
    17 begin
    18 
    18 
    19 ML_file "Tools/typechk.ML"
    19 ML_file "Tools/typechk.ML"
    20 
    20