# HG changeset patch # User wenzelm # Date 1444509897 -7200 # Node ID 045b4d7a53e291410bd1e64a4bf4ef365eea643f # Parent 808222c1cf662ef9efab04a95c27d1037e661987 tuned syntax -- more symbols; diff -r 808222c1cf66 -r 045b4d7a53e2 src/ZF/Order.thy --- a/src/ZF/Order.thy Sat Oct 10 22:44:45 2015 +0200 +++ b/src/ZF/Order.thy Sat Oct 10 22:44:57 2015 +0200 @@ -49,8 +49,8 @@ {f \ A->B. \x\A. \y\A. :r \ :s}" definition - ord_iso :: "[i,i,i,i]=>i" (*Order isomorphisms*) where - "ord_iso(A,r,B,s) == + ord_iso :: "[i,i,i,i]=>i" ("(\_, _\ \/ \_, _\)" 51) (*Order isomorphisms*) where + "\A,r\ \ \B,s\ == {f \ bij(A,B). \x\A. \y\A. :r \ :s}" definition @@ -66,11 +66,6 @@ first :: "[i, i, i] => o" where "first(u, X, R) == u \ X & (\v\X. v\u \ \ R)" - -notation (xsymbols) - ord_iso ("(\_, _\ \/ \_, _\)" 51) - - subsection\Immediate Consequences of the Definitions\ lemma part_ord_Imp_asym: