src/ZF/Ordinal.thy
changeset 61378 3e04c9ca001a
parent 60770 240563fbf41d
child 61397 6204c86280ff
equal deleted inserted replaced
61377:517feb558c77 61378:3e04c9ca001a
    30 abbreviation
    30 abbreviation
    31   le  (infixl "le" 50) where
    31   le  (infixl "le" 50) where
    32   "x le y == x < succ(y)"
    32   "x le y == x < succ(y)"
    33 
    33 
    34 notation (xsymbols)
    34 notation (xsymbols)
    35   le  (infixl "\<le>" 50)
       
    36 
       
    37 notation (HTML output)
       
    38   le  (infixl "\<le>" 50)
    35   le  (infixl "\<le>" 50)
    39 
    36 
    40 
    37 
    41 subsection\<open>Rules for Transset\<close>
    38 subsection\<open>Rules for Transset\<close>
    42 
    39