src/ZF/Order.thy
changeset 16417 9bc16273c2d4
parent 13701 0a9228532106
child 24893 b8ef7afe3a6b
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     7         by Kenneth Kunen.  Chapter 1, section 6.
     7         by Kenneth Kunen.  Chapter 1, section 6.
     8 *)
     8 *)
     9 
     9 
    10 header{*Partial and Total Orderings: Basic Definitions and Properties*}
    10 header{*Partial and Total Orderings: Basic Definitions and Properties*}
    11 
    11 
    12 theory Order = WF + Perm:
    12 theory Order imports WF Perm begin
    13 
    13 
    14 constdefs
    14 constdefs
    15 
    15 
    16   part_ord :: "[i,i]=>o"          	(*Strict partial ordering*)
    16   part_ord :: "[i,i]=>o"          	(*Strict partial ordering*)
    17    "part_ord(A,r) == irrefl(A,r) & trans[A](r)"
    17    "part_ord(A,r) == irrefl(A,r) & trans[A](r)"