src/ZF/QPair.thy
changeset 16417 9bc16273c2d4
parent 14854 61bdf2ae4dc5
child 17782 b3846df9d643
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     9     is not a limit ordinal? 
     9     is not a limit ordinal? 
    10 *)
    10 *)
    11 
    11 
    12 header{*Quine-Inspired Ordered Pairs and Disjoint Sums*}
    12 header{*Quine-Inspired Ordered Pairs and Disjoint Sums*}
    13 
    13 
    14 theory QPair = Sum + func:
    14 theory QPair imports Sum func begin
    15 
    15 
    16 text{*For non-well-founded data
    16 text{*For non-well-founded data
    17 structures in ZF.  Does not precisely follow Quine's construction.  Thanks
    17 structures in ZF.  Does not precisely follow Quine's construction.  Thanks
    18 to Thomas Forster for suggesting this approach!
    18 to Thomas Forster for suggesting this approach!
    19 
    19