src/HOL/Tools/Function/induction_schema.ML
changeset 55642 63beb38e9258
parent 54742 7a86358a3c0b
child 55968 94242fa87638
--- a/src/HOL/Tools/Function/induction_schema.ML	Fri Feb 21 00:09:55 2014 +0100
+++ b/src/HOL/Tools/Function/induction_schema.ML	Fri Feb 21 00:09:56 2014 +0100
@@ -44,7 +44,7 @@
 fun meta thm = thm RS eq_reflection
 
 fun sum_prod_conv ctxt = Raw_Simplifier.rewrite ctxt true
-  (map meta (@{thm split_conv} :: @{thms sum.cases}))
+  (map meta (@{thm split_conv} :: @{thms sum.case}))
 
 fun term_conv thy cv t =
   cv (cterm_of thy t)
@@ -315,7 +315,7 @@
         val Pxs = cert (HOLogic.mk_Trueprop (P_comp $ x))
           |> Goal.init
           |> (Simplifier.rewrite_goals_tac ctxt
-                (map meta (branch_hyp :: @{thm split_conv} :: @{thms sum.cases}))
+                (map meta (branch_hyp :: @{thm split_conv} :: @{thms sum.case}))
               THEN CONVERSION (ind_rulify ctxt) 1)
           |> Seq.hd
           |> Thm.elim_implies (Conv.fconv_rule Drule.beta_eta_conversion bstep)