src/HOL/Algebra/FiniteProduct.thy
changeset 44890 22f665a2e91c
parent 41433 1b8ff770f02c
child 46721 f88b187ad8ca
--- a/src/HOL/Algebra/FiniteProduct.thy	Sun Sep 11 22:56:05 2011 +0200
+++ b/src/HOL/Algebra/FiniteProduct.thy	Mon Sep 12 07:55:43 2011 +0200
@@ -171,7 +171,7 @@
     (EX y. (A, y) \<in> foldSetD D f e & v = f x y)"
   apply auto
   apply (rule_tac A1 = A in finite_imp_foldSetD [THEN exE])
-     apply (fastsimp dest: foldSetD_imp_finite)
+     apply (fastforce dest: foldSetD_imp_finite)
     apply assumption
    apply assumption
   apply (blast intro: foldSetD_determ)
@@ -328,7 +328,7 @@
            apply fast
           apply fast
          apply assumption
-        apply (fastsimp intro: m_closed)
+        apply (fastforce intro: m_closed)
        apply simp+
    apply fast
   apply (auto simp add: finprod_def)
@@ -431,13 +431,13 @@
       next
         assume "x ~: B" "!!i. i \<in> insert x B \<Longrightarrow> f i = g i"
           "g \<in> insert x B \<rightarrow> carrier G"
-        thus "f \<in> B -> carrier G" by fastsimp
+        thus "f \<in> B -> carrier G" by fastforce
       next
         assume "x ~: B" "!!i. i \<in> insert x B \<Longrightarrow> f i = g i"
           "g \<in> insert x B \<rightarrow> carrier G"
-        thus "f x \<in> carrier G" by fastsimp
+        thus "f x \<in> carrier G" by fastforce
       qed
-      also from insert have "... = g x \<otimes> finprod G g B" by fastsimp
+      also from insert have "... = g x \<otimes> finprod G g B" by fastforce
       also from insert have "... = finprod G g (insert x B)"
       by (intro finprod_insert [THEN sym]) auto
       finally show ?case .