# HG changeset patch # User wenzelm # Date 1181810328 -7200 # Node ID 5460951833fa35196d0f38200d4f7f95d96189d0 # Parent 0459ab90389a475f1af5752aa33395eba01ffbad tuned proofs: avoid implicit prems; diff -r 0459ab90389a -r 5460951833fa src/HOL/Algebra/AbelCoset.thy --- a/src/HOL/Algebra/AbelCoset.thy Thu Jun 14 09:54:14 2007 +0200 +++ b/src/HOL/Algebra/AbelCoset.thy Thu Jun 14 10:38:48 2007 +0200 @@ -712,7 +712,7 @@ and repr: "H +> x = H +> y" shows "y \ H +> x" by (rule group.repr_independenceD [OF a_group a_subgroup, - folded a_r_coset_def, simplified monoid_record_simps]) + folded a_r_coset_def, simplified monoid_record_simps]) (rule ycarr, rule repr) subsection {* Lemmas for the Set of Right Cosets *} @@ -731,7 +731,7 @@ and Bcarr: "B \ carrier G" shows "A <+> B \ carrier G" by (rule monoid.set_mult_closed [OF a_monoid, - folded set_add_def, simplified monoid_record_simps]) + folded set_add_def, simplified monoid_record_simps]) (rule Acarr, rule Bcarr) lemma (in abelian_group) add_additive_subgroups: assumes subH: "additive_subgroup H G" diff -r 0459ab90389a -r 5460951833fa src/HOL/Algebra/Ideal.thy --- a/src/HOL/Algebra/Ideal.thy Thu Jun 14 09:54:14 2007 +0200 +++ b/src/HOL/Algebra/Ideal.thy Thu Jun 14 10:38:48 2007 +0200 @@ -67,7 +67,7 @@ lemma (in maximalideal) is_maximalideal: shows "maximalideal I R" -by - +by fact lemma maximalidealI: includes ideal @@ -673,17 +673,9 @@ lemma (in ideal) primeidealCE: includes cring assumes notprime: "\ primeideal I R" - and elim1: "carrier R = I \ P" - and elim2: "(\a b. a \ carrier R \ b \ carrier R \ a \ b \ I \ a \ I \ b \ I) \ P" - shows "P" -proof - - from notprime - have "carrier R = I \ (\a b. a \ carrier R \ b \ carrier R \ a \ b \ I \ a \ I \ b \ I)" - by (intro primeidealCD) - thus "P" - apply (rule disjE) - by (erule elim1, erule elim2) -qed + obtains "carrier R = I" + | "\a b. a \ carrier R \ b \ carrier R \ a \ b \ I \ a \ I \ b \ I" + using primeidealCD [OF R.is_cring notprime] by blast text {* If @{text "{\}"} is a prime ideal of a commutative ring, the ring is a domain *} lemma (in cring) zeroprimeideal_domainI: @@ -790,21 +782,21 @@ by fast def J \ "{x\carrier R. a \ x \ I}" - from acarr - have idealJ: "ideal J R" by (unfold J_def, intro helper_max_prime) + from R.is_cring and acarr + have idealJ: "ideal J R" unfolding J_def by (rule helper_max_prime) have IsubJ: "I \ J" proof fix x assume xI: "x \ I" from this and acarr - have "a \ x \ I" by (intro I_l_closed) + have "a \ x \ I" by (intro I_l_closed) from xI[THEN a_Hcarr] this - show "x \ J" by (unfold J_def, fast) + show "x \ J" unfolding J_def by fast qed from abI and acarr bcarr - have "b \ J" by (unfold J_def, fast) + have "b \ J" unfolding J_def by fast from bnI and this have JnI: "J \ I" by fast from acarr @@ -812,7 +804,7 @@ from this and anI have "a \ \ \ I" by simp from one_closed and this - have "\ \ J" by (unfold J_def, fast) + have "\ \ J" unfolding J_def by fast hence Jncarr: "J \ carrier R" by fast interpret ideal ["J" "R"] by (rule idealJ)