removed cases_of;
renamed cases_tac to case_tac; tuned to work with basic HOL as well;
add_cases_induct: proper case names;
adapted to new PureThy.add_thms etc.;
Exor = Main +
constdefs
exor :: bool => bool => bool
"exor A B == (A & ~B) | (~A & B)"
end