recovered old version of simple_induct; split the main function into small functions
theory Ind_Code
imports "../Base" Simple_Inductive_Package
begin
text {*
@{ML_chunk [display,gray] induction_rules}
*}
text {*
@{ML_chunk [display,gray] intro_rules}
*}
end