- Moved abs_def to drule.ML
- elim_defs now takes a boolean argument which controls the automatic
expansion of theorems mentioning constants whose definitions are
eliminated
ConstDefs = Types +
constdefs nand :: gate
"nand A B == ~(A & B)"
exor :: gate
"exor A B == A & ~B | ~A & B"
end