src/HOL/intr_elim.ML
changeset 2688 889a1cbd1aca
parent 2414 13df7d6c5c3b
child 3978 7e1cfed19d94
equal deleted inserted replaced
2687:b7c86d3c9d0a 2688:889a1cbd1aca
   142                   (unfold RS Ind_Syntax.equals_CollectD);
   142                   (unfold RS Ind_Syntax.equals_CollectD);
   143 
   143 
   144   (*String s should have the form t:Si where Si is an inductive set*)
   144   (*String s should have the form t:Si where Si is an inductive set*)
   145   fun mk_cases defs s = 
   145   fun mk_cases defs s = 
   146       rule_by_tactic (con_elim_tac defs)
   146       rule_by_tactic (con_elim_tac defs)
   147         (assume_read Inductive.thy s  RS  elim);
   147           (assume_read Inductive.thy s  RS  elim) 
       
   148       |> standard;
   148 
   149 
   149   val raw_induct = standard ([big_rec_def, mono] MRS Fp.induct)
   150   val raw_induct = standard ([big_rec_def, mono] MRS Fp.induct)
   150   and rec_names = rec_names
   151   and rec_names = rec_names
   151   end
   152   end
   152 end;
   153 end;