diff -r 00f8be1b7209 -r f87c8c449018 src/ZF/Order.thy --- a/src/ZF/Order.thy Thu Aug 24 00:55:42 2000 +0200 +++ b/src/ZF/Order.thy Thu Aug 24 11:05:20 2000 +0200 @@ -35,12 +35,15 @@ ord_iso_map_def "ord_iso_map(A,r,B,s) == - UN x:A. UN y:B. UN f: ord_iso(pred(A,x,r), r, pred(B,y,s), s). - {}" + UN x:A. UN y:B. UN f: ord_iso(pred(A,x,r), r, pred(B,y,s), s). {}" constdefs first :: [i, i, i] => o "first(u, X, R) == u:X & (ALL v:X. v~=u --> : R)" +syntax (xsymbols) + ord_iso :: [i,i,i,i]=>i ("('(_,_') \\ '(_,_'))" 50) + + end