# HG changeset patch # User wenzelm # Date 1315080325 -7200 # Node ID 3fb27b19e058e41923a6fe0b4a4e6e875a1e275f # Parent 7de87f1ae96533ca4edf1c45d00652642969cff7 misc tuning and simplification of proofs; diff -r 7de87f1ae965 -r 3fb27b19e058 src/HOL/Algebra/Ideal.thy --- a/src/HOL/Algebra/Ideal.thy Sat Sep 03 21:15:35 2011 +0200 +++ b/src/HOL/Algebra/Ideal.thy Sat Sep 03 22:05:25 2011 +0200 @@ -14,25 +14,24 @@ locale ideal = additive_subgroup I R + ring R for I and R (structure) + assumes I_l_closed: "\a \ I; x \ carrier R\ \ x \ a \ I" - and I_r_closed: "\a \ I; x \ carrier R\ \ a \ x \ I" + and I_r_closed: "\a \ I; x \ carrier R\ \ a \ x \ I" sublocale ideal \ abelian_subgroup I R -apply (intro abelian_subgroupI3 abelian_group.intro) - apply (rule ideal.axioms, rule ideal_axioms) - apply (rule abelian_group.axioms, rule ring.axioms, rule ideal.axioms, rule ideal_axioms) -apply (rule abelian_group.axioms, rule ring.axioms, rule ideal.axioms, rule ideal_axioms) -done + apply (intro abelian_subgroupI3 abelian_group.intro) + apply (rule ideal.axioms, rule ideal_axioms) + apply (rule abelian_group.axioms, rule ring.axioms, rule ideal.axioms, rule ideal_axioms) + apply (rule abelian_group.axioms, rule ring.axioms, rule ideal.axioms, rule ideal_axioms) + done -lemma (in ideal) is_ideal: - "ideal I R" -by (rule ideal_axioms) +lemma (in ideal) is_ideal: "ideal I R" + by (rule ideal_axioms) lemma idealI: fixes R (structure) assumes "ring R" assumes a_subgroup: "subgroup I \carrier = carrier R, mult = add R, one = zero R\" - and I_l_closed: "\a x. \a \ I; x \ carrier R\ \ x \ a \ I" - and I_r_closed: "\a x. \a \ I; x \ carrier R\ \ a \ x \ I" + and I_l_closed: "\a x. \a \ I; x \ carrier R\ \ x \ a \ I" + and I_r_closed: "\a x. \a \ I; x \ carrier R\ \ a \ x \ I" shows "ideal I R" proof - interpret ring R by fact @@ -47,19 +46,16 @@ subsubsection (in ring) {* Ideals Generated by a Subset of @{term "carrier R"} *} -definition - genideal :: "('a, 'b) ring_scheme \ 'a set \ 'a set" ("Idl\ _" [80] 79) +definition genideal :: "_ \ 'a set \ 'a set" ("Idl\ _" [80] 79) where "genideal R S = Inter {I. ideal I R \ S \ I}" - subsubsection {* Principal Ideals *} locale principalideal = ideal + assumes generate: "\i \ carrier R. I = Idl {i}" -lemma (in principalideal) is_principalideal: - shows "principalideal I R" -by (rule principalideal_axioms) +lemma (in principalideal) is_principalideal: "principalideal I R" + by (rule principalideal_axioms) lemma principalidealI: fixes R (structure) @@ -68,7 +64,9 @@ shows "principalideal I R" proof - interpret ideal I R by fact - show ?thesis by (intro principalideal.intro principalideal_axioms.intro) (rule is_ideal, rule generate) + show ?thesis + by (intro principalideal.intro principalideal_axioms.intro) + (rule is_ideal, rule generate) qed @@ -76,22 +74,22 @@ locale maximalideal = ideal + assumes I_notcarr: "carrier R \ I" - and I_maximal: "\ideal J R; I \ J; J \ carrier R\ \ J = I \ J = carrier R" + and I_maximal: "\ideal J R; I \ J; J \ carrier R\ \ J = I \ J = carrier R" -lemma (in maximalideal) is_maximalideal: - shows "maximalideal I R" -by (rule maximalideal_axioms) +lemma (in maximalideal) is_maximalideal: "maximalideal I R" + by (rule maximalideal_axioms) lemma maximalidealI: fixes R assumes "ideal I R" assumes I_notcarr: "carrier R \ I" - and I_maximal: "\J. \ideal J R; I \ J; J \ carrier R\ \ J = I \ J = carrier R" + and I_maximal: "\J. \ideal J R; I \ J; J \ carrier R\ \ J = I \ J = carrier R" shows "maximalideal I R" proof - interpret ideal I R by fact - show ?thesis by (intro maximalideal.intro maximalideal_axioms.intro) - (rule is_ideal, rule I_notcarr, rule I_maximal) + show ?thesis + by (intro maximalideal.intro maximalideal_axioms.intro) + (rule is_ideal, rule I_notcarr, rule I_maximal) qed @@ -99,24 +97,24 @@ locale primeideal = ideal + cring + assumes I_notcarr: "carrier R \ I" - and I_prime: "\a \ carrier R; b \ carrier R; a \ b \ I\ \ a \ I \ b \ I" + and I_prime: "\a \ carrier R; b \ carrier R; a \ b \ I\ \ a \ I \ b \ I" -lemma (in primeideal) is_primeideal: - shows "primeideal I R" -by (rule primeideal_axioms) +lemma (in primeideal) is_primeideal: "primeideal I R" + by (rule primeideal_axioms) lemma primeidealI: fixes R (structure) assumes "ideal I R" assumes "cring R" assumes I_notcarr: "carrier R \ I" - and I_prime: "\a b. \a \ carrier R; b \ carrier R; a \ b \ I\ \ a \ I \ b \ I" + and I_prime: "\a b. \a \ carrier R; b \ carrier R; a \ b \ I\ \ a \ I \ b \ I" shows "primeideal I R" proof - interpret ideal I R by fact interpret cring R by fact - show ?thesis by (intro primeideal.intro primeideal_axioms.intro) - (rule is_ideal, rule is_cring, rule I_notcarr, rule I_prime) + show ?thesis + by (intro primeideal.intro primeideal_axioms.intro) + (rule is_ideal, rule is_cring, rule I_notcarr, rule I_prime) qed lemma primeidealI2: @@ -124,9 +122,9 @@ assumes "additive_subgroup I R" assumes "cring R" assumes I_l_closed: "\a x. \a \ I; x \ carrier R\ \ x \ a \ I" - and I_r_closed: "\a x. \a \ I; x \ carrier R\ \ a \ x \ I" - and I_notcarr: "carrier R \ I" - and I_prime: "\a b. \a \ carrier R; b \ carrier R; a \ b \ I\ \ a \ I \ b \ I" + and I_r_closed: "\a x. \a \ I; x \ carrier R\ \ a \ x \ I" + and I_notcarr: "carrier R \ I" + and I_prime: "\a b. \a \ carrier R; b \ carrier R; a \ b \ I\ \ a \ I \ b \ I" shows "primeideal I R" proof - interpret additive_subgroup I R by fact @@ -144,31 +142,27 @@ subsection {* Special Ideals *} -lemma (in ring) zeroideal: - shows "ideal {\} R" -apply (intro idealI subgroup.intro) - apply (rule is_ring) - apply simp+ - apply (fold a_inv_def, simp) - apply simp+ -done +lemma (in ring) zeroideal: "ideal {\} R" + apply (intro idealI subgroup.intro) + apply (rule is_ring) + apply simp+ + apply (fold a_inv_def, simp) + apply simp+ + done -lemma (in ring) oneideal: - shows "ideal (carrier R) R" +lemma (in ring) oneideal: "ideal (carrier R) R" by (rule idealI) (auto intro: is_ring add.subgroupI) -lemma (in "domain") zeroprimeideal: - shows "primeideal {\} R" -apply (intro primeidealI) - apply (rule zeroideal) - apply (rule domain.axioms, rule domain_axioms) - defer 1 - apply (simp add: integral) +lemma (in "domain") zeroprimeideal: "primeideal {\} R" + apply (intro primeidealI) + apply (rule zeroideal) + apply (rule domain.axioms, rule domain_axioms) + defer 1 + apply (simp add: integral) proof (rule ccontr, simp) assume "carrier R = {\}" - from this have "\ = \" by (rule one_zeroI) - from this and one_not_zero - show "False" by simp + then have "\ = \" by (rule one_zeroI) + with one_not_zero show False by simp qed @@ -177,22 +171,20 @@ lemma (in ideal) one_imp_carrier: assumes I_one_closed: "\ \ I" shows "I = carrier R" -apply (rule) -apply (rule) -apply (rule a_Hcarr, simp) + apply (rule) + apply (rule) + apply (rule a_Hcarr, simp) proof fix x assume xcarr: "x \ carrier R" - from I_one_closed and this - have "x \ \ \ I" by (intro I_l_closed) - from this and xcarr - show "x \ I" by simp + with I_one_closed have "x \ \ \ I" by (intro I_l_closed) + with xcarr show "x \ I" by simp qed lemma (in ideal) Icarr: assumes iI: "i \ I" shows "i \ carrier R" -using iI by (rule a_Hcarr) + using iI by (rule a_Hcarr) subsection {* Intersection of Ideals *} @@ -207,17 +199,17 @@ interpret ideal I R by fact interpret ideal J R by fact show ?thesis -apply (intro idealI subgroup.intro) - apply (rule is_ring) - apply (force simp add: a_subset) - apply (simp add: a_inv_def[symmetric]) - apply simp - apply (simp add: a_inv_def[symmetric]) - apply (clarsimp, rule) - apply (fast intro: ideal.I_l_closed ideal.intro assms)+ -apply (clarsimp, rule) - apply (fast intro: ideal.I_r_closed ideal.intro assms)+ -done + apply (intro idealI subgroup.intro) + apply (rule is_ring) + apply (force simp add: a_subset) + apply (simp add: a_inv_def[symmetric]) + apply simp + apply (simp add: a_inv_def[symmetric]) + apply (clarsimp, rule) + apply (fast intro: ideal.I_l_closed ideal.intro assms)+ + apply (clarsimp, rule) + apply (fast intro: ideal.I_r_closed ideal.intro assms)+ + done qed text {* The intersection of any Number of Ideals is again @@ -226,26 +218,25 @@ assumes Sideals: "\I. I \ S \ ideal I R" and notempty: "S \ {}" shows "ideal (Inter S) R" -apply (unfold_locales) -apply (simp_all add: Inter_eq) - apply rule unfolding mem_Collect_eq defer 1 - apply rule defer 1 - apply rule defer 1 - apply (fold a_inv_def, rule) defer 1 - apply rule defer 1 - apply rule defer 1 + apply (unfold_locales) + apply (simp_all add: Inter_eq) + apply rule unfolding mem_Collect_eq defer 1 + apply rule defer 1 + apply rule defer 1 + apply (fold a_inv_def, rule) defer 1 + apply rule defer 1 + apply rule defer 1 proof - fix x y assume "\I\S. x \ I" - hence xI: "\I. I \ S \ x \ I" by simp + then have xI: "\I. I \ S \ x \ I" by simp assume "\I\S. y \ I" - hence yI: "\I. I \ S \ y \ I" by simp + then have yI: "\I. I \ S \ y \ I" by simp fix J assume JS: "J \ S" interpret ideal J R by (rule Sideals[OF JS]) - from xI[OF JS] and yI[OF JS] - show "x \ y \ J" by (rule a_closed) + from xI[OF JS] and yI[OF JS] show "x \ y \ J" by (rule a_closed) next fix J assume JS: "J \ S" @@ -254,50 +245,47 @@ next fix x assume "\I\S. x \ I" - hence xI: "\I. I \ S \ x \ I" by simp + then have xI: "\I. I \ S \ x \ I" by simp fix J assume JS: "J \ S" interpret ideal J R by (rule Sideals[OF JS]) - from xI[OF JS] - show "\ x \ J" by (rule a_inv_closed) + from xI[OF JS] show "\ x \ J" by (rule a_inv_closed) next fix x y assume "\I\S. x \ I" - hence xI: "\I. I \ S \ x \ I" by simp + then have xI: "\I. I \ S \ x \ I" by simp assume ycarr: "y \ carrier R" fix J assume JS: "J \ S" interpret ideal J R by (rule Sideals[OF JS]) - from xI[OF JS] and ycarr - show "y \ x \ J" by (rule I_l_closed) + from xI[OF JS] and ycarr show "y \ x \ J" by (rule I_l_closed) next fix x y assume "\I\S. x \ I" - hence xI: "\I. I \ S \ x \ I" by simp + then have xI: "\I. I \ S \ x \ I" by simp assume ycarr: "y \ carrier R" fix J assume JS: "J \ S" interpret ideal J R by (rule Sideals[OF JS]) - from xI[OF JS] and ycarr - show "x \ y \ J" by (rule I_r_closed) + from xI[OF JS] and ycarr show "x \ y \ J" by (rule I_r_closed) next fix x assume "\I\S. x \ I" - hence xI: "\I. I \ S \ x \ I" by simp + then have xI: "\I. I \ S \ x \ I" by simp from notempty have "\I0. I0 \ S" by blast - from this obtain I0 where I0S: "I0 \ S" by auto + then obtain I0 where I0S: "I0 \ S" by auto interpret ideal I0 R by (rule Sideals[OF I0S]) from xI[OF I0S] have "x \ I0" . - from this and a_subset show "x \ carrier R" by fast + with a_subset show "x \ carrier R" by fast next qed @@ -309,40 +297,41 @@ assumes idealI: "ideal I R" and idealJ: "ideal J R" shows "ideal (I <+> J) R" -apply (rule ideal.intro) - apply (rule add_additive_subgroups) - apply (intro ideal.axioms[OF idealI]) - apply (intro ideal.axioms[OF idealJ]) - apply (rule is_ring) -apply (rule ideal_axioms.intro) - apply (simp add: set_add_defs, clarsimp) defer 1 - apply (simp add: set_add_defs, clarsimp) defer 1 + apply (rule ideal.intro) + apply (rule add_additive_subgroups) + apply (intro ideal.axioms[OF idealI]) + apply (intro ideal.axioms[OF idealJ]) + apply (rule is_ring) + apply (rule ideal_axioms.intro) + apply (simp add: set_add_defs, clarsimp) defer 1 + apply (simp add: set_add_defs, clarsimp) defer 1 proof - fix x i j assume xcarr: "x \ carrier R" - and iI: "i \ I" - and jJ: "j \ J" + and iI: "i \ I" + and jJ: "j \ J" from xcarr ideal.Icarr[OF idealI iI] ideal.Icarr[OF idealJ jJ] - have c: "(i \ j) \ x = (i \ x) \ (j \ x)" by algebra - from xcarr and iI - have a: "i \ x \ I" by (simp add: ideal.I_r_closed[OF idealI]) - from xcarr and jJ - have b: "j \ x \ J" by (simp add: ideal.I_r_closed[OF idealJ]) - from a b c - show "\ha\I. \ka\J. (i \ j) \ x = ha \ ka" by fast + have c: "(i \ j) \ x = (i \ x) \ (j \ x)" + by algebra + from xcarr and iI have a: "i \ x \ I" + by (simp add: ideal.I_r_closed[OF idealI]) + from xcarr and jJ have b: "j \ x \ J" + by (simp add: ideal.I_r_closed[OF idealJ]) + from a b c show "\ha\I. \ka\J. (i \ j) \ x = ha \ ka" + by fast next fix x i j assume xcarr: "x \ carrier R" - and iI: "i \ I" - and jJ: "j \ J" + and iI: "i \ I" + and jJ: "j \ J" from xcarr ideal.Icarr[OF idealI iI] ideal.Icarr[OF idealJ jJ] - have c: "x \ (i \ j) = (x \ i) \ (x \ j)" by algebra - from xcarr and iI - have a: "x \ i \ I" by (simp add: ideal.I_l_closed[OF idealI]) - from xcarr and jJ - have b: "x \ j \ J" by (simp add: ideal.I_l_closed[OF idealJ]) - from a b c - show "\ha\I. \ka\J. x \ (i \ j) = ha \ ka" by fast + have c: "x \ (i \ j) = (x \ i) \ (x \ j)" by algebra + from xcarr and iI have a: "x \ i \ I" + by (simp add: ideal.I_l_closed[OF idealI]) + from xcarr and jJ have b: "x \ j \ J" + by (simp add: ideal.I_l_closed[OF idealJ]) + from a b c show "\ha\I. \ka\J. x \ (i \ j) = ha \ ka" + by fast qed @@ -361,87 +350,74 @@ lemma (in ring) genideal_self: assumes "S \ carrier R" shows "S \ Idl S" -unfolding genideal_def -by fast + unfolding genideal_def by fast lemma (in ring) genideal_self': assumes carr: "i \ carrier R" shows "i \ Idl {i}" proof - - from carr - have "{i} \ Idl {i}" by (fast intro!: genideal_self) - thus "i \ Idl {i}" by fast + from carr have "{i} \ Idl {i}" by (fast intro!: genideal_self) + then show "i \ Idl {i}" by fast qed text {* @{term genideal} generates the minimal ideal *} lemma (in ring) genideal_minimal: assumes a: "ideal I R" - and b: "S \ I" + and b: "S \ I" shows "Idl S \ I" -unfolding genideal_def -by (rule, elim InterD, simp add: a b) + unfolding genideal_def by rule (elim InterD, simp add: a b) text {* Generated ideals and subsets *} lemma (in ring) Idl_subset_ideal: assumes Iideal: "ideal I R" - and Hcarr: "H \ carrier R" + and Hcarr: "H \ carrier R" shows "(Idl H \ I) = (H \ I)" proof assume a: "Idl H \ I" from Hcarr have "H \ Idl H" by (rule genideal_self) - from this and a - show "H \ I" by simp + with a show "H \ I" by simp next fix x assume HI: "H \ I" - - from Iideal and HI - have "I \ {I. ideal I R \ H \ I}" by fast - from this - show "Idl H \ I" - unfolding genideal_def - by fast + from Iideal and HI have "I \ {I. ideal I R \ H \ I}" by fast + then show "Idl H \ I" unfolding genideal_def by fast qed lemma (in ring) subset_Idl_subset: assumes Icarr: "I \ carrier R" - and HI: "H \ I" + and HI: "H \ I" shows "Idl H \ Idl I" proof - - from HI and genideal_self[OF Icarr] - have HIdlI: "H \ Idl I" by fast + from HI and genideal_self[OF Icarr] have HIdlI: "H \ Idl I" + by fast - from Icarr - have Iideal: "ideal (Idl I) R" by (rule genideal_ideal) - from HI and Icarr - have "H \ carrier R" by fast - from Iideal and this - have "(H \ Idl I) = (Idl H \ Idl I)" - by (rule Idl_subset_ideal[symmetric]) + from Icarr have Iideal: "ideal (Idl I) R" + by (rule genideal_ideal) + from HI and Icarr have "H \ carrier R" + by fast + with Iideal have "(H \ Idl I) = (Idl H \ Idl I)" + by (rule Idl_subset_ideal[symmetric]) - from HIdlI and this - show "Idl H \ Idl I" by simp + with HIdlI show "Idl H \ Idl I" by simp qed lemma (in ring) Idl_subset_ideal': assumes acarr: "a \ carrier R" and bcarr: "b \ carrier R" shows "(Idl {a} \ Idl {b}) = (a \ Idl {b})" -apply (subst Idl_subset_ideal[OF genideal_ideal[of "{b}"], of "{a}"]) - apply (fast intro: bcarr, fast intro: acarr) -apply fast -done + apply (subst Idl_subset_ideal[OF genideal_ideal[of "{b}"], of "{a}"]) + apply (fast intro: bcarr, fast intro: acarr) + apply fast + done -lemma (in ring) genideal_zero: - "Idl {\} = {\}" -apply rule - apply (rule genideal_minimal[OF zeroideal], simp) -apply (simp add: genideal_self') -done +lemma (in ring) genideal_zero: "Idl {\} = {\}" + apply rule + apply (rule genideal_minimal[OF zeroideal], simp) + apply (simp add: genideal_self') + done -lemma (in ring) genideal_one: - "Idl {\} = carrier R" +lemma (in ring) genideal_one: "Idl {\} = carrier R" proof - - interpret ideal "Idl {\}" "R" by (rule genideal_ideal, fast intro: one_closed) + interpret ideal "Idl {\}" "R" by (rule genideal_ideal) fast show "Idl {\} = carrier R" apply (rule, rule a_subset) apply (simp add: one_imp_carrier genideal_self') @@ -451,77 +427,76 @@ text {* Generation of Principal Ideals in Commutative Rings *} -definition - cgenideal :: "('a, 'b) monoid_scheme \ 'a \ 'a set" ("PIdl\ _" [80] 79) +definition cgenideal :: "_ \ 'a \ 'a set" ("PIdl\ _" [80] 79) where "cgenideal R a = {x \\<^bsub>R\<^esub> a | x. x \ carrier R}" text {* genhideal (?) really generates an ideal *} lemma (in cring) cgenideal_ideal: assumes acarr: "a \ carrier R" shows "ideal (PIdl a) R" -apply (unfold cgenideal_def) -apply (rule idealI[OF is_ring]) - apply (rule subgroup.intro) - apply (simp_all add: monoid_record_simps) - apply (blast intro: acarr m_closed) - apply clarsimp defer 1 - defer 1 - apply (fold a_inv_def, clarsimp) defer 1 - apply clarsimp defer 1 - apply clarsimp defer 1 + apply (unfold cgenideal_def) + apply (rule idealI[OF is_ring]) + apply (rule subgroup.intro) + apply simp_all + apply (blast intro: acarr) + apply clarsimp defer 1 + defer 1 + apply (fold a_inv_def, clarsimp) defer 1 + apply clarsimp defer 1 + apply clarsimp defer 1 proof - fix x y assume xcarr: "x \ carrier R" - and ycarr: "y \ carrier R" + and ycarr: "y \ carrier R" note carr = acarr xcarr ycarr - from carr - have "x \ a \ y \ a = (x \ y) \ a" by (simp add: l_distr) - from this and carr - show "\z. x \ a \ y \ a = z \ a \ z \ carrier R" by fast + from carr have "x \ a \ y \ a = (x \ y) \ a" + by (simp add: l_distr) + with carr show "\z. x \ a \ y \ a = z \ a \ z \ carrier R" + by fast next from l_null[OF acarr, symmetric] and zero_closed - show "\x. \ = x \ a \ x \ carrier R" by fast + show "\x. \ = x \ a \ x \ carrier R" by fast next fix x assume xcarr: "x \ carrier R" note carr = acarr xcarr - from carr - have "\ (x \ a) = (\ x) \ a" by (simp add: l_minus) - from this and carr - show "\z. \ (x \ a) = z \ a \ z \ carrier R" by fast + from carr have "\ (x \ a) = (\ x) \ a" + by (simp add: l_minus) + with carr show "\z. \ (x \ a) = z \ a \ z \ carrier R" + by fast next fix x y assume xcarr: "x \ carrier R" and ycarr: "y \ carrier R" note carr = acarr xcarr ycarr - from carr - have "y \ a \ x = (y \ x) \ a" by (simp add: m_assoc, simp add: m_comm) - from this and carr - show "\z. y \ a \ x = z \ a \ z \ carrier R" by fast + from carr have "y \ a \ x = (y \ x) \ a" + by (simp add: m_assoc) (simp add: m_comm) + with carr show "\z. y \ a \ x = z \ a \ z \ carrier R" + by fast next fix x y assume xcarr: "x \ carrier R" and ycarr: "y \ carrier R" note carr = acarr xcarr ycarr - from carr - have "x \ (y \ a) = (x \ y) \ a" by (simp add: m_assoc) - from this and carr - show "\z. x \ (y \ a) = z \ a \ z \ carrier R" by fast + from carr have "x \ (y \ a) = (x \ y) \ a" + by (simp add: m_assoc) + with carr show "\z. x \ (y \ a) = z \ a \ z \ carrier R" + by fast qed lemma (in ring) cgenideal_self: assumes icarr: "i \ carrier R" shows "i \ PIdl i" -unfolding cgenideal_def + unfolding cgenideal_def proof simp - from icarr - have "i = \ \ i" by simp - from this and icarr - show "\x. i = x \ i \ x \ carrier R" by fast + from icarr have "i = \ \ i" + by simp + with icarr show "\x. i = x \ i \ x \ carrier R" + by fast qed text {* @{const "cgenideal"} is minimal *} @@ -532,7 +507,8 @@ shows "PIdl a \ J" proof - interpret ideal J R by fact - show ?thesis unfolding cgenideal_def + show ?thesis + unfolding cgenideal_def apply rule apply clarify using aJ @@ -543,30 +519,28 @@ lemma (in cring) cgenideal_eq_genideal: assumes icarr: "i \ carrier R" shows "PIdl i = Idl {i}" -apply rule - apply (intro cgenideal_minimal) - apply (rule genideal_ideal, fast intro: icarr) - apply (rule genideal_self', fast intro: icarr) -apply (intro genideal_minimal) - apply (rule cgenideal_ideal [OF icarr]) -apply (simp, rule cgenideal_self [OF icarr]) -done + apply rule + apply (intro cgenideal_minimal) + apply (rule genideal_ideal, fast intro: icarr) + apply (rule genideal_self', fast intro: icarr) + apply (intro genideal_minimal) + apply (rule cgenideal_ideal [OF icarr]) + apply (simp, rule cgenideal_self [OF icarr]) + done -lemma (in cring) cgenideal_eq_rcos: - "PIdl i = carrier R #> i" -unfolding cgenideal_def r_coset_def -by fast +lemma (in cring) cgenideal_eq_rcos: "PIdl i = carrier R #> i" + unfolding cgenideal_def r_coset_def by fast lemma (in cring) cgenideal_is_principalideal: assumes icarr: "i \ carrier R" shows "principalideal (PIdl i) R" -apply (rule principalidealI) -apply (rule cgenideal_ideal [OF icarr]) + apply (rule principalidealI) + apply (rule cgenideal_ideal [OF icarr]) proof - - from icarr - have "PIdl i = Idl {i}" by (rule cgenideal_eq_genideal) - from icarr and this - show "\i'\carrier R. PIdl i = Idl {i'}" by fast + from icarr have "PIdl i = Idl {i}" + by (rule cgenideal_eq_genideal) + with icarr show "\i'\carrier R. PIdl i = Idl {i'}" + by fast qed @@ -574,83 +548,79 @@ lemma (in ring) union_genideal: assumes idealI: "ideal I R" - and idealJ: "ideal J R" + and idealJ: "ideal J R" shows "Idl (I \ J) = I <+> J" -apply rule - apply (rule ring.genideal_minimal) - apply (rule is_ring) - apply (rule add_ideals[OF idealI idealJ]) - apply (rule) - apply (simp add: set_add_defs) apply (elim disjE) defer 1 defer 1 - apply (rule) apply (simp add: set_add_defs genideal_def) apply clarsimp defer 1 + apply rule + apply (rule ring.genideal_minimal) + apply (rule is_ring) + apply (rule add_ideals[OF idealI idealJ]) + apply (rule) + apply (simp add: set_add_defs) apply (elim disjE) defer 1 defer 1 + apply (rule) apply (simp add: set_add_defs genideal_def) apply clarsimp defer 1 proof - fix x assume xI: "x \ I" have ZJ: "\ \ J" - by (intro additive_subgroup.zero_closed, rule ideal.axioms[OF idealJ]) - from ideal.Icarr[OF idealI xI] - have "x = x \ \" by algebra - from xI and ZJ and this - show "\h\I. \k\J. x = h \ k" by fast + by (intro additive_subgroup.zero_closed) (rule ideal.axioms[OF idealJ]) + from ideal.Icarr[OF idealI xI] have "x = x \ \" + by algebra + with xI and ZJ show "\h\I. \k\J. x = h \ k" + by fast next fix x assume xJ: "x \ J" have ZI: "\ \ I" - by (intro additive_subgroup.zero_closed, rule ideal.axioms[OF idealI]) - from ideal.Icarr[OF idealJ xJ] - have "x = \ \ x" by algebra - from ZI and xJ and this - show "\h\I. \k\J. x = h \ k" by fast + by (intro additive_subgroup.zero_closed, rule ideal.axioms[OF idealI]) + from ideal.Icarr[OF idealJ xJ] have "x = \ \ x" + by algebra + with ZI and xJ show "\h\I. \k\J. x = h \ k" + by fast next fix i j K assume iI: "i \ I" - and jJ: "j \ J" - and idealK: "ideal K R" - and IK: "I \ K" - and JK: "J \ K" - from iI and IK - have iK: "i \ K" by fast - from jJ and JK - have jK: "j \ K" by fast - from iK and jK - show "i \ j \ K" by (intro additive_subgroup.a_closed) (rule ideal.axioms[OF idealK]) + and jJ: "j \ J" + and idealK: "ideal K R" + and IK: "I \ K" + and JK: "J \ K" + from iI and IK have iK: "i \ K" by fast + from jJ and JK have jK: "j \ K" by fast + from iK and jK show "i \ j \ K" + by (intro additive_subgroup.a_closed) (rule ideal.axioms[OF idealK]) qed subsection {* Properties of Principal Ideals *} text {* @{text "\"} generates the zero ideal *} -lemma (in ring) zero_genideal: - shows "Idl {\} = {\}" -apply rule -apply (simp add: genideal_minimal zeroideal) -apply (fast intro!: genideal_self) -done +lemma (in ring) zero_genideal: "Idl {\} = {\}" + apply rule + apply (simp add: genideal_minimal zeroideal) + apply (fast intro!: genideal_self) + done text {* @{text "\"} generates the unit ideal *} -lemma (in ring) one_genideal: - shows "Idl {\} = carrier R" +lemma (in ring) one_genideal: "Idl {\} = carrier R" proof - - have "\ \ Idl {\}" by (simp add: genideal_self') - thus "Idl {\} = carrier R" by (intro ideal.one_imp_carrier, fast intro: genideal_ideal) + have "\ \ Idl {\}" + by (simp add: genideal_self') + then show "Idl {\} = carrier R" + by (intro ideal.one_imp_carrier) (fast intro: genideal_ideal) qed text {* The zero ideal is a principal ideal *} -corollary (in ring) zeropideal: - shows "principalideal {\} R" -apply (rule principalidealI) - apply (rule zeroideal) -apply (blast intro!: zero_closed zero_genideal[symmetric]) -done +corollary (in ring) zeropideal: "principalideal {\} R" + apply (rule principalidealI) + apply (rule zeroideal) + apply (blast intro!: zero_genideal[symmetric]) + done text {* The unit ideal is a principal ideal *} -corollary (in ring) onepideal: - shows "principalideal (carrier R) R" -apply (rule principalidealI) - apply (rule oneideal) -apply (blast intro!: one_closed one_genideal[symmetric]) -done +corollary (in ring) onepideal: "principalideal (carrier R) R" + apply (rule principalidealI) + apply (rule oneideal) + apply (blast intro!: one_genideal[symmetric]) + done text {* Every principal ideal is a right coset of the carrier *} @@ -659,28 +629,24 @@ shows "\x\I. I = carrier R #> x" proof - interpret cring R by fact - from generate - obtain i - where icarr: "i \ carrier R" - and I1: "I = Idl {i}" - by fast+ + from generate obtain i where icarr: "i \ carrier R" and I1: "I = Idl {i}" + by fast+ - from icarr and genideal_self[of "{i}"] - have "i \ Idl {i}" by fast - hence iI: "i \ I" by (simp add: I1) + from icarr and genideal_self[of "{i}"] have "i \ Idl {i}" + by fast + then have iI: "i \ I" by (simp add: I1) - from I1 icarr - have I2: "I = PIdl i" by (simp add: cgenideal_eq_genideal) + from I1 icarr have I2: "I = PIdl i" + by (simp add: cgenideal_eq_genideal) have "PIdl i = carrier R #> i" - unfolding cgenideal_def r_coset_def - by fast + unfolding cgenideal_def r_coset_def by fast - from I2 and this - have "I = carrier R #> i" by simp + with I2 have "I = carrier R #> i" + by simp - from iI and this - show "\x\I. I = carrier R #> x" by fast + with iI show "\x\I. I = carrier R #> x" + by fast qed @@ -693,16 +659,16 @@ proof (rule ccontr, clarsimp) interpret cring R by fact assume InR: "carrier R \ I" - and "\a. a \ carrier R \ (\b. a \ b \ I \ b \ carrier R \ a \ I \ b \ I)" - hence I_prime: "\ a b. \a \ carrier R; b \ carrier R; a \ b \ I\ \ a \ I \ b \ I" by simp + and "\a. a \ carrier R \ (\b. a \ b \ I \ b \ carrier R \ a \ I \ b \ I)" + then have I_prime: "\ a b. \a \ carrier R; b \ carrier R; a \ b \ I\ \ a \ I \ b \ I" + by simp have "primeideal I R" - apply (rule primeideal.intro [OF is_ideal is_cring]) - apply (rule primeideal_axioms.intro) - apply (rule InR) - apply (erule (2) I_prime) - done - from this and notprime - show "False" by simp + apply (rule primeideal.intro [OF is_ideal is_cring]) + apply (rule primeideal_axioms.intro) + apply (rule InR) + apply (erule (2) I_prime) + done + with notprime show False by simp qed lemma (in ideal) primeidealCE: @@ -721,47 +687,44 @@ lemma (in cring) zeroprimeideal_domainI: assumes pi: "primeideal {\} R" shows "domain R" -apply (rule domain.intro, rule is_cring) -apply (rule domain_axioms.intro) + apply (rule domain.intro, rule is_cring) + apply (rule domain_axioms.intro) proof (rule ccontr, simp) interpret primeideal "{\}" "R" by (rule pi) assume "\ = \" - hence "carrier R = {\}" by (rule one_zeroD) - from this[symmetric] and I_notcarr - show "False" by simp + then have "carrier R = {\}" by (rule one_zeroD) + from this[symmetric] and I_notcarr show False + by simp next interpret primeideal "{\}" "R" by (rule pi) fix a b - assume ab: "a \ b = \" - and carr: "a \ carrier R" "b \ carrier R" - from ab - have abI: "a \ b \ {\}" by fast - from carr and this - have "a \ {\} \ b \ {\}" by (rule I_prime) - thus "a = \ \ b = \" by simp + assume ab: "a \ b = \" and carr: "a \ carrier R" "b \ carrier R" + from ab have abI: "a \ b \ {\}" + by fast + with carr have "a \ {\} \ b \ {\}" + by (rule I_prime) + then show "a = \ \ b = \" by simp qed -corollary (in cring) domain_eq_zeroprimeideal: - shows "domain R = primeideal {\} R" -apply rule - apply (erule domain.zeroprimeideal) -apply (erule zeroprimeideal_domainI) -done +corollary (in cring) domain_eq_zeroprimeideal: "domain R = primeideal {\} R" + apply rule + apply (erule domain.zeroprimeideal) + apply (erule zeroprimeideal_domainI) + done subsection {* Maximal Ideals *} lemma (in ideal) helper_I_closed: assumes carr: "a \ carrier R" "x \ carrier R" "y \ carrier R" - and axI: "a \ x \ I" + and axI: "a \ x \ I" shows "a \ (x \ y) \ I" proof - - from axI and carr - have "(a \ x) \ y \ I" by (simp add: I_r_closed) - also from carr - have "(a \ x) \ y = a \ (x \ y)" by (simp add: m_assoc) - finally - show "a \ (x \ y) \ I" . + from axI and carr have "(a \ x) \ y \ I" + by (simp add: I_r_closed) + also from carr have "(a \ x) \ y = a \ (x \ y)" + by (simp add: m_assoc) + finally show "a \ (x \ y) \ I" . qed lemma (in ideal) helper_max_prime: @@ -787,19 +750,18 @@ have "\(a \ x) \ I" by simp also from acarr xcarr have "\(a \ x) = a \ (\x)" by algebra - finally - show "a \ (\x) \ I" . - from acarr - have "a \ \ = \" by simp + finally show "a \ (\x) \ I" . + from acarr have "a \ \ = \" by simp next fix x y assume xcarr: "x \ carrier R" and ycarr: "y \ carrier R" and ayI: "a \ y \ I" - from ayI and acarr xcarr ycarr - have "a \ (y \ x) \ I" by (simp add: helper_I_closed) - moreover from xcarr ycarr - have "y \ x = x \ y" by (simp add: m_comm) + from ayI and acarr xcarr ycarr have "a \ (y \ x) \ I" + by (simp add: helper_I_closed) + moreover + from xcarr ycarr have "y \ x = x \ y" + by (simp add: m_comm) ultimately show "a \ (x \ y) \ I" by simp qed @@ -818,40 +780,36 @@ apply (simp add: I_notcarr) proof - assume "\a b. a \ carrier R \ b \ carrier R \ a \ b \ I \ a \ I \ b \ I" - from this - obtain a b - where acarr: "a \ carrier R" - and bcarr: "b \ carrier R" - and abI: "a \ b \ I" - and anI: "a \ I" - and bnI: "b \ I" - by fast + then obtain a b where + acarr: "a \ carrier R" and + bcarr: "b \ carrier R" and + abI: "a \ b \ I" and + anI: "a \ I" and + bnI: "b \ I" by fast def J \ "{x\carrier R. a \ x \ I}" - from is_cring and acarr - have idealJ: "ideal J R" unfolding J_def by (rule helper_max_prime) + from 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) - from xI[THEN a_Hcarr] this - show "x \ J" unfolding J_def by fast + with acarr have "a \ x \ I" + by (intro I_l_closed) + with xI[THEN a_Hcarr] show "x \ J" + unfolding J_def by fast qed - from abI and acarr bcarr - have "b \ J" unfolding J_def by fast - from bnI and this - have JnI: "J \ I" by fast + from abI and acarr bcarr have "b \ J" + unfolding J_def by fast + with bnI have JnI: "J \ I" by fast from acarr have "a = a \ \" by algebra - from this and anI - have "a \ \ \ I" by simp - from one_closed and this - have "\ \ J" unfolding J_def by fast - hence Jncarr: "J \ carrier R" by fast + with anI have "a \ \ \ I" by simp + with one_closed have "\ \ J" + unfolding J_def by fast + then have Jncarr: "J \ carrier R" by fast interpret ideal J R by (rule idealJ) @@ -862,8 +820,7 @@ apply (rule a_subset) done - from this and JnI and Jncarr - show "False" by simp + with JnI and Jncarr show False by simp qed qed @@ -873,111 +830,93 @@ --"A non-zero cring that has only the two trivial ideals is a field" lemma (in cring) trivialideals_fieldI: assumes carrnzero: "carrier R \ {\}" - and haveideals: "{I. ideal I R} = {{\}, carrier R}" + and haveideals: "{I. ideal I R} = {{\}, carrier R}" shows "field R" -apply (rule cring_fieldI) -apply (rule, rule, rule) - apply (erule Units_closed) -defer 1 - apply rule -defer 1 + apply (rule cring_fieldI) + apply (rule, rule, rule) + apply (erule Units_closed) + defer 1 + apply rule + defer 1 proof (rule ccontr, simp) assume zUnit: "\ \ Units R" - hence a: "\ \ inv \ = \" by (rule Units_r_inv) - from zUnit - have "\ \ inv \ = \" by (intro l_null, rule Units_inv_closed) - from a[symmetric] and this - have "\ = \" by simp - hence "carrier R = {\}" by (rule one_zeroD) - from this and carrnzero - show "False" by simp + then have a: "\ \ inv \ = \" by (rule Units_r_inv) + from zUnit have "\ \ inv \ = \" + by (intro l_null) (rule Units_inv_closed) + with a[symmetric] have "\ = \" by simp + then have "carrier R = {\}" by (rule one_zeroD) + with carrnzero show False by simp next fix x assume xcarr': "x \ carrier R - {\}" - hence xcarr: "x \ carrier R" by fast - from xcarr' - have xnZ: "x \ \" by fast - from xcarr - have xIdl: "ideal (PIdl x) R" by (intro cgenideal_ideal, fast) + then have xcarr: "x \ carrier R" by fast + from xcarr' have xnZ: "x \ \" by fast + from xcarr have xIdl: "ideal (PIdl x) R" + by (intro cgenideal_ideal) fast - from xcarr - have "x \ PIdl x" by (intro cgenideal_self, fast) - from this and xnZ - have "PIdl x \ {\}" by fast - from haveideals and this - have "PIdl x = carrier R" - by (blast intro!: xIdl) - hence "\ \ PIdl x" by simp - hence "\y. \ = y \ x \ y \ carrier R" unfolding cgenideal_def by blast - from this - obtain y - where ycarr: " y \ carrier R" - and ylinv: "\ = y \ x" - by fast+ - from ylinv and xcarr ycarr - have yrinv: "\ = x \ y" by (simp add: m_comm) + from xcarr have "x \ PIdl x" + by (intro cgenideal_self) fast + with xnZ have "PIdl x \ {\}" by fast + with haveideals have "PIdl x = carrier R" + by (blast intro!: xIdl) + then have "\ \ PIdl x" by simp + then have "\y. \ = y \ x \ y \ carrier R" + unfolding cgenideal_def by blast + then obtain y where ycarr: " y \ carrier R" and ylinv: "\ = y \ x" + by fast+ + from ylinv and xcarr ycarr have yrinv: "\ = x \ y" + by (simp add: m_comm) from ycarr and ylinv[symmetric] and yrinv[symmetric] - have "\y \ carrier R. y \ x = \ \ x \ y = \" by fast - from this and xcarr - show "x \ Units R" - unfolding Units_def - by fast + have "\y \ carrier R. y \ x = \ \ x \ y = \" by fast + with xcarr show "x \ Units R" + unfolding Units_def by fast qed -lemma (in field) all_ideals: - shows "{I. ideal I R} = {{\}, carrier R}" -apply (rule, rule) +lemma (in field) all_ideals: "{I. ideal I R} = {{\}, carrier R}" + apply (rule, rule) proof - fix I assume a: "I \ {I. ideal I R}" - with this - interpret ideal I R by simp + then interpret ideal I R by simp show "I \ {{\}, carrier R}" proof (cases "\a. a \ I - {\}") - assume "\a. a \ I - {\}" - from this - obtain a - where aI: "a \ I" - and anZ: "a \ \" - by fast+ - from aI[THEN a_Hcarr] anZ - have aUnit: "a \ Units R" by (simp add: field_Units) - hence a: "a \ inv a = \" by (rule Units_r_inv) - from aI and aUnit - have "a \ inv a \ I" by (simp add: I_r_closed del: Units_r_inv) - hence oneI: "\ \ I" by (simp add: a[symmetric]) + case True + then obtain a where aI: "a \ I" and anZ: "a \ \" + by fast+ + from aI[THEN a_Hcarr] anZ have aUnit: "a \ Units R" + by (simp add: field_Units) + then have a: "a \ inv a = \" by (rule Units_r_inv) + from aI and aUnit have "a \ inv a \ I" + by (simp add: I_r_closed del: Units_r_inv) + then have oneI: "\ \ I" by (simp add: a[symmetric]) have "carrier R \ I" proof fix x assume xcarr: "x \ carrier R" - from oneI and this - have "\ \ x \ I" by (rule I_r_closed) - from this and xcarr - show "x \ I" by simp + with oneI have "\ \ x \ I" by (rule I_r_closed) + with xcarr show "x \ I" by simp qed - from this and a_subset - have "I = carrier R" by fast - thus "I \ {{\}, carrier R}" by fast + with a_subset have "I = carrier R" by fast + then show "I \ {{\}, carrier R}" by fast next - assume "\ (\a. a \ I - {\})" - hence IZ: "\a. a \ I \ a = \" by simp + case False + then have IZ: "\a. a \ I \ a = \" by simp have a: "I \ {\}" proof fix x assume "x \ I" - hence "x = \" by (rule IZ) - thus "x \ {\}" by fast + then have "x = \" by (rule IZ) + then show "x \ {\}" by fast qed have "\ \ I" by simp - hence "{\} \ I" by fast + then have "{\} \ I" by fast - from this and a - have "I = {\}" by fast - thus "I \ {{\}, carrier R}" by fast + with a have "I = {\}" by fast + then show "I \ {{\}, carrier R}" by fast qed qed (simp add: zeroideal oneideal) @@ -985,52 +924,47 @@ lemma (in cring) trivialideals_eq_field: assumes carrnzero: "carrier R \ {\}" shows "({I. ideal I R} = {{\}, carrier R}) = field R" -by (fast intro!: trivialideals_fieldI[OF carrnzero] field.all_ideals) + by (fast intro!: trivialideals_fieldI[OF carrnzero] field.all_ideals) text {* Like zeroprimeideal for domains *} -lemma (in field) zeromaximalideal: - "maximalideal {\} R" -apply (rule maximalidealI) - apply (rule zeroideal) +lemma (in field) zeromaximalideal: "maximalideal {\} R" + apply (rule maximalidealI) + apply (rule zeroideal) proof- - from one_not_zero - have "\ \ {\}" by simp - from this and one_closed - show "carrier R \ {\}" by fast + from one_not_zero have "\ \ {\}" by simp + with one_closed show "carrier R \ {\}" by fast next fix J assume Jideal: "ideal J R" - hence "J \ {I. ideal I R}" - by fast - - from this and all_ideals - show "J = {\} \ J = carrier R" by simp + then have "J \ {I. ideal I R}" by fast + with all_ideals show "J = {\} \ J = carrier R" + by simp qed lemma (in cring) zeromaximalideal_fieldI: assumes zeromax: "maximalideal {\} R" shows "field R" -apply (rule trivialideals_fieldI, rule maximalideal.I_notcarr[OF zeromax]) -apply rule apply clarsimp defer 1 - apply (simp add: zeroideal oneideal) + apply (rule trivialideals_fieldI, rule maximalideal.I_notcarr[OF zeromax]) + apply rule apply clarsimp defer 1 + apply (simp add: zeroideal oneideal) proof - fix J assume Jn0: "J \ {\}" - and idealJ: "ideal J R" + and idealJ: "ideal J R" interpret ideal J R by (rule idealJ) - have "{\} \ J" by (rule ccontr, simp) + have "{\} \ J" by (rule ccontr) simp from zeromax and idealJ and this and a_subset - have "J = {\} \ J = carrier R" by (rule maximalideal.I_maximal) - from this and Jn0 - show "J = carrier R" by simp + have "J = {\} \ J = carrier R" + by (rule maximalideal.I_maximal) + with Jn0 show "J = carrier R" + by simp qed -lemma (in cring) zeromaximalideal_eq_field: - "maximalideal {\} R = field R" -apply rule - apply (erule zeromaximalideal_fieldI) -apply (erule field.zeromaximalideal) -done +lemma (in cring) zeromaximalideal_eq_field: "maximalideal {\} R = field R" + apply rule + apply (erule zeromaximalideal_fieldI) + apply (erule field.zeromaximalideal) + done end diff -r 7de87f1ae965 -r 3fb27b19e058 src/HOL/Algebra/Ring.thy --- a/src/HOL/Algebra/Ring.thy Sat Sep 03 21:15:35 2011 +0200 +++ b/src/HOL/Algebra/Ring.thy Sat Sep 03 22:05:25 2011 +0200 @@ -367,7 +367,7 @@ proof - assume R: "x \ carrier R" "y \ carrier R" then have "(\ x) \ y \ x \ y = (\ x \ x) \ y" by (simp add: l_distr) - also from R have "... = \" by (simp add: l_neg l_null) + also from R have "... = \" by (simp add: l_neg) finally have "(\ x) \ y \ x \ y = \" . with R have "(\ x) \ y \ x \ y \ \ (x \ y) = \ \ \ (x \ y)" by simp with R show ?thesis by (simp add: a_assoc r_neg) @@ -378,7 +378,7 @@ proof - assume R: "x \ carrier R" "y \ carrier R" then have "x \ (\ y) \ x \ y = x \ (\ y \ y)" by (simp add: r_distr) - also from R have "... = \" by (simp add: l_neg r_null) + also from R have "... = \" by (simp add: l_neg) finally have "x \ (\ y) \ x \ y = \" . with R have "x \ (\ y) \ x \ y \ \ (x \ y) = \ \ \ (x \ y)" by simp with R show ?thesis by (simp add: a_assoc r_neg ) @@ -464,7 +464,6 @@ proof - interpret ring R by fact interpret cring S by fact -ML_val {* Algebra.print_structures @{context} *} from RS show ?thesis by algebra qed