Added setup for simplification of equality constraints in cases rules.
authorberghofe
Sat, 30 Jan 2010 16:59:49 +0100
changeset 34988 cca208c8d619
parent 34987 c1e8af37ee75
child 34989 b5c6e59e2cd7
Added setup for simplification of equality constraints in cases rules.
src/HOL/HOL.thy
--- a/src/HOL/HOL.thy	Sat Jan 30 16:58:46 2010 +0100
+++ b/src/HOL/HOL.thy	Sat Jan 30 16:59:49 2010 +0100
@@ -1453,6 +1453,7 @@
   val atomize = @{thms induct_atomize}
   val rulify = @{thms induct_rulify'}
   val rulify_fallback = @{thms induct_rulify_fallback}
+  val equal_def = @{thm induct_equal_def}
   fun dest_def (Const (@{const_name induct_equal}, _) $ t $ u) = SOME (t, u)
     | dest_def _ = NONE
   val trivial_tac = match_tac @{thms induct_trueI}