Removing the datatype declaration of "order" allows the standard General.order
to be used. Thus we can use Int.compare and String.compare instead of the
slower home-grown versions.
Exor = Main +
constdefs
exor :: bool => bool => bool
"exor A B == (A & ~B) | (~A & B)"
end