src/HOL/Tools/function_package/mutual.ML
changeset 22526 be2269950fe5
parent 22497 1fe951654cee
child 22567 1565d476a9e2
--- a/src/HOL/Tools/function_package/mutual.ML	Mon Mar 26 14:54:45 2007 +0200
+++ b/src/HOL/Tools/function_package/mutual.ML	Mon Mar 26 16:35:33 2007 +0200
@@ -261,7 +261,7 @@
                  (HOLogic.Trueprop $ HOLogic.mk_eq (list_comb (f, args), rhs))
                  (fn _ => SIMPSET (unfold_tac all_orig_fdefs)
                           THEN EqSubst.eqsubst_tac ctxt [0] [simp] 1
-                          THEN SIMPSET' simp_tac 1)
+                          THEN SIMPSET' (fn ss => simp_tac (ss addsimps [@{thm "lproj_inl"}, @{thm "rproj_inr"}])) 1)
         |> restore_cond 
         |> export
     end