first stage in tidying up Real and Hyperreal.
Factor cancellation simprocs
inverse #0 = #0
simprules for division
corrected ambigous syntax definitions in Hyperreal
Exor = Main +constdefs exor :: bool => bool => bool"exor A B == (A & ~B) | (~A & B)"end