src/HOL/Algebra/Ideal.thy
author wenzelm
Sun, 12 Aug 2018 14:28:28 +0200
changeset 68743 91162dd89571
parent 68604 57721285d4ef
child 68687 2976a4a3b126
permissions -rw-r--r--
proper session dirs;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
41959
b460124855b8 tuned headers;
wenzelm
parents: 41433
diff changeset
     1
(*  Title:      HOL/Algebra/Ideal.thy
35849
b5522b51cb1e standard headers;
wenzelm
parents: 35848
diff changeset
     2
    Author:     Stephan Hohe, TU Muenchen
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
     3
*)
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
     4
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
     5
theory Ideal
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
     6
imports Ring AbelCoset
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
     7
begin
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
     8
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
     9
section \<open>Ideals\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    10
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
    11
subsection \<open>Definitions\<close>
27717
21bbd410ba04 Generalised polynomial lemmas from cring to ring.
ballarin
parents: 27714
diff changeset
    12
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
    13
subsubsection \<open>General definition\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    14
29240
bb81c3709fb6 More porting to new locales.
ballarin
parents: 29237
diff changeset
    15
locale ideal = additive_subgroup I R + ring R for I and R (structure) +
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    16
  assumes I_l_closed: "\<lbrakk>a \<in> I; x \<in> carrier R\<rbrakk> \<Longrightarrow> x \<otimes> a \<in> I"
68445
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
    17
      and I_r_closed: "\<lbrakk>a \<in> I; x \<in> carrier R\<rbrakk> \<Longrightarrow> a \<otimes> x \<in> I"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    18
29237
e90d9d51106b More porting to new locales.
ballarin
parents: 27717
diff changeset
    19
sublocale ideal \<subseteq> abelian_subgroup I R
68458
023b353911c5 Algebra tidy-up
paulson <lp15@cam.ac.uk>
parents: 68445
diff changeset
    20
proof (intro abelian_subgroupI3 abelian_group.intro)
023b353911c5 Algebra tidy-up
paulson <lp15@cam.ac.uk>
parents: 68445
diff changeset
    21
  show "additive_subgroup I R"
023b353911c5 Algebra tidy-up
paulson <lp15@cam.ac.uk>
parents: 68445
diff changeset
    22
    by (simp add: is_additive_subgroup)
023b353911c5 Algebra tidy-up
paulson <lp15@cam.ac.uk>
parents: 68445
diff changeset
    23
  show "abelian_monoid R"
023b353911c5 Algebra tidy-up
paulson <lp15@cam.ac.uk>
parents: 68445
diff changeset
    24
    by (simp add: abelian_monoid_axioms)
023b353911c5 Algebra tidy-up
paulson <lp15@cam.ac.uk>
parents: 68445
diff changeset
    25
  show "abelian_group_axioms R"
023b353911c5 Algebra tidy-up
paulson <lp15@cam.ac.uk>
parents: 68445
diff changeset
    26
    using abelian_group_def is_abelian_group by blast
023b353911c5 Algebra tidy-up
paulson <lp15@cam.ac.uk>
parents: 68445
diff changeset
    27
qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    28
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
    29
lemma (in ideal) is_ideal: "ideal I R"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
    30
  by (rule ideal_axioms)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    31
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    32
lemma idealI:
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
    33
  fixes R (structure)
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
    34
  assumes "ring R"
68443
43055b016688 New material from Martin Baillon and Paulo Emílio de Vilhena
paulson <lp15@cam.ac.uk>
parents: 67443
diff changeset
    35
  assumes a_subgroup: "subgroup I (add_monoid R)"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
    36
    and I_l_closed: "\<And>a x. \<lbrakk>a \<in> I; x \<in> carrier R\<rbrakk> \<Longrightarrow> x \<otimes> a \<in> I"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
    37
    and I_r_closed: "\<And>a x. \<lbrakk>a \<in> I; x \<in> carrier R\<rbrakk> \<Longrightarrow> a \<otimes> x \<in> I"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    38
  shows "ideal I R"
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
    39
proof -
29237
e90d9d51106b More porting to new locales.
ballarin
parents: 27717
diff changeset
    40
  interpret ring R by fact
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
    41
  show ?thesis  
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
    42
    by (auto simp: ideal.intro ideal_axioms.intro additive_subgroupI a_subgroup is_ring I_l_closed I_r_closed)
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
    43
qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    44
35849
b5522b51cb1e standard headers;
wenzelm
parents: 35848
diff changeset
    45
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
    46
subsubsection (in ring) \<open>Ideals Generated by a Subset of @{term "carrier R"}\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    47
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
    48
definition genideal :: "_ \<Rightarrow> 'a set \<Rightarrow> 'a set"  ("Idl\<index> _" [80] 79)
61952
546958347e05 prefer symbols for "Union", "Inter";
wenzelm
parents: 61506
diff changeset
    49
  where "genideal R S = \<Inter>{I. ideal I R \<and> S \<subseteq> I}"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    50
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
    51
subsubsection \<open>Principal Ideals\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    52
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    53
locale principalideal = ideal +
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    54
  assumes generate: "\<exists>i \<in> carrier R. I = Idl {i}"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    55
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
    56
lemma (in principalideal) is_principalideal: "principalideal I R"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
    57
  by (rule principalideal_axioms)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    58
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    59
lemma principalidealI:
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
    60
  fixes R (structure)
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
    61
  assumes "ideal I R"
47409
c5be1120980d tuned proofs;
wenzelm
parents: 44677
diff changeset
    62
    and generate: "\<exists>i \<in> carrier R. I = Idl {i}"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    63
  shows "principalideal I R"
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
    64
proof -
29237
e90d9d51106b More porting to new locales.
ballarin
parents: 27717
diff changeset
    65
  interpret ideal I R by fact
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
    66
  show ?thesis
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
    67
    by (intro principalideal.intro principalideal_axioms.intro)
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
    68
      (rule is_ideal, rule generate)
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
    69
qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    70
35849
b5522b51cb1e standard headers;
wenzelm
parents: 35848
diff changeset
    71
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
    72
subsubsection \<open>Maximal Ideals\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    73
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    74
locale maximalideal = ideal +
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    75
  assumes I_notcarr: "carrier R \<noteq> I"
68445
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
    76
    and I_maximal: "\<lbrakk>ideal J R; I \<subseteq> J; J \<subseteq> carrier R\<rbrakk> \<Longrightarrow> (J = I) \<or> (J = carrier R)"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    77
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
    78
lemma (in maximalideal) is_maximalideal: "maximalideal I R"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
    79
  by (rule maximalideal_axioms)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    80
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    81
lemma maximalidealI:
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
    82
  fixes R
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
    83
  assumes "ideal I R"
47409
c5be1120980d tuned proofs;
wenzelm
parents: 44677
diff changeset
    84
    and I_notcarr: "carrier R \<noteq> I"
68445
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
    85
    and I_maximal: "\<And>J. \<lbrakk>ideal J R; I \<subseteq> J; J \<subseteq> carrier R\<rbrakk> \<Longrightarrow> (J = I) \<or> (J = carrier R)"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    86
  shows "maximalideal I R"
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
    87
proof -
29237
e90d9d51106b More porting to new locales.
ballarin
parents: 27717
diff changeset
    88
  interpret ideal I R by fact
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
    89
  show ?thesis
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
    90
    by (intro maximalideal.intro maximalideal_axioms.intro)
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
    91
      (rule is_ideal, rule I_notcarr, rule I_maximal)
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
    92
qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    93
35849
b5522b51cb1e standard headers;
wenzelm
parents: 35848
diff changeset
    94
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
    95
subsubsection \<open>Prime Ideals\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    96
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    97
locale primeideal = ideal + cring +
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
    98
  assumes I_notcarr: "carrier R \<noteq> I"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
    99
    and I_prime: "\<lbrakk>a \<in> carrier R; b \<in> carrier R; a \<otimes> b \<in> I\<rbrakk> \<Longrightarrow> a \<in> I \<or> b \<in> I"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   100
63633
2accfb71e33b is_prime -> prime
eberlm <eberlm@in.tum.de>
parents: 63167
diff changeset
   101
lemma (in primeideal) primeideal: "primeideal I R"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   102
  by (rule primeideal_axioms)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   103
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   104
lemma primeidealI:
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   105
  fixes R (structure)
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   106
  assumes "ideal I R"
47409
c5be1120980d tuned proofs;
wenzelm
parents: 44677
diff changeset
   107
    and "cring R"
c5be1120980d tuned proofs;
wenzelm
parents: 44677
diff changeset
   108
    and I_notcarr: "carrier R \<noteq> I"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   109
    and I_prime: "\<And>a b. \<lbrakk>a \<in> carrier R; b \<in> carrier R; a \<otimes> b \<in> I\<rbrakk> \<Longrightarrow> a \<in> I \<or> b \<in> I"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   110
  shows "primeideal I R"
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   111
proof -
29237
e90d9d51106b More porting to new locales.
ballarin
parents: 27717
diff changeset
   112
  interpret ideal I R by fact
e90d9d51106b More porting to new locales.
ballarin
parents: 27717
diff changeset
   113
  interpret cring R by fact
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   114
  show ?thesis
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   115
    by (intro primeideal.intro primeideal_axioms.intro)
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   116
      (rule is_ideal, rule is_cring, rule I_notcarr, rule I_prime)
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   117
qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   118
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   119
lemma primeidealI2:
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   120
  fixes R (structure)
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   121
  assumes "additive_subgroup I R"
47409
c5be1120980d tuned proofs;
wenzelm
parents: 44677
diff changeset
   122
    and "cring R"
c5be1120980d tuned proofs;
wenzelm
parents: 44677
diff changeset
   123
    and I_l_closed: "\<And>a x. \<lbrakk>a \<in> I; x \<in> carrier R\<rbrakk> \<Longrightarrow> x \<otimes> a \<in> I"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   124
    and I_r_closed: "\<And>a x. \<lbrakk>a \<in> I; x \<in> carrier R\<rbrakk> \<Longrightarrow> a \<otimes> x \<in> I"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   125
    and I_notcarr: "carrier R \<noteq> I"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   126
    and I_prime: "\<And>a b. \<lbrakk>a \<in> carrier R; b \<in> carrier R; a \<otimes> b \<in> I\<rbrakk> \<Longrightarrow> a \<in> I \<or> b \<in> I"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   127
  shows "primeideal I R"
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   128
proof -
29240
bb81c3709fb6 More porting to new locales.
ballarin
parents: 29237
diff changeset
   129
  interpret additive_subgroup I R by fact
29237
e90d9d51106b More porting to new locales.
ballarin
parents: 27717
diff changeset
   130
  interpret cring R by fact
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   131
  show ?thesis apply intro_locales
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   132
    apply (intro ideal_axioms.intro)
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   133
    apply (erule (1) I_l_closed)
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   134
    apply (erule (1) I_r_closed)
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   135
    by (simp add: I_notcarr I_prime primeideal_axioms.intro)
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   136
qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   137
35849
b5522b51cb1e standard headers;
wenzelm
parents: 35848
diff changeset
   138
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   139
subsection \<open>Special Ideals\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   140
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   141
lemma (in ring) zeroideal: "ideal {\<zero>} R"
68445
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   142
  by (intro idealI subgroup.intro) (simp_all add: is_ring)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   143
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   144
lemma (in ring) oneideal: "ideal (carrier R) R"
41433
1b8ff770f02c Abelian group facts obtained from group facts via interpretation (sublocale).
ballarin
parents: 35849
diff changeset
   145
  by (rule idealI) (auto intro: is_ring add.subgroupI)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   146
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   147
lemma (in "domain") zeroprimeideal: "primeideal {\<zero>} R"
68445
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   148
proof -
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   149
  have "carrier R \<noteq> {\<zero>}"
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   150
    by (simp add: carrier_one_not_zero)
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   151
  then show ?thesis
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   152
    by (metis (no_types, lifting) domain_axioms domain_def integral primeidealI singleton_iff zeroideal)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   153
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   154
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   155
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   156
subsection \<open>General Ideal Properies\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   157
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   158
lemma (in ideal) one_imp_carrier:
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   159
  assumes I_one_closed: "\<one> \<in> I"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   160
  shows "I = carrier R"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   161
proof
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   162
  show "carrier R \<subseteq> I"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   163
    using I_r_closed assms by fastforce
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   164
  show "I \<subseteq> carrier R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   165
    by (rule a_subset)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   166
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   167
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   168
lemma (in ideal) Icarr:
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   169
  assumes iI: "i \<in> I"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   170
  shows "i \<in> carrier R"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   171
  using iI by (rule a_Hcarr)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   172
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   173
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   174
subsection \<open>Intersection of Ideals\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   175
61506
wenzelm
parents: 61382
diff changeset
   176
paragraph \<open>Intersection of two ideals\<close>
wenzelm
parents: 61382
diff changeset
   177
text \<open>The intersection of any two ideals is again an ideal in @{term R}\<close>
wenzelm
parents: 61382
diff changeset
   178
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   179
lemma (in ring) i_intersect:
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   180
  assumes "ideal I R"
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   181
  assumes "ideal J R"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   182
  shows "ideal (I \<inter> J) R"
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   183
proof -
29237
e90d9d51106b More porting to new locales.
ballarin
parents: 27717
diff changeset
   184
  interpret ideal I R by fact
29240
bb81c3709fb6 More porting to new locales.
ballarin
parents: 29237
diff changeset
   185
  interpret ideal J R by fact
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   186
  have IJ: "I \<inter> J \<subseteq> carrier R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   187
    by (force simp: a_subset)
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   188
  show ?thesis
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   189
    apply (intro idealI subgroup.intro)
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   190
    apply (simp_all add: IJ is_ring I_l_closed assms ideal.I_l_closed ideal.I_r_closed flip: a_inv_def)
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   191
    done
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   192
qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   193
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   194
text \<open>The intersection of any Number of Ideals is again an Ideal in @{term R}\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   195
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   196
lemma (in ring) i_Intersect:
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   197
  assumes Sideals: "\<And>I. I \<in> S \<Longrightarrow> ideal I R" and notempty: "S \<noteq> {}"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   198
  shows "ideal (\<Inter>S) R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   199
proof -
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   200
  { fix x y J
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   201
    assume "\<forall>I\<in>S. x \<in> I" "\<forall>I\<in>S. y \<in> I" and JS: "J \<in> S"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   202
    interpret ideal J R by (rule Sideals[OF JS])
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   203
    have "x \<oplus> y \<in> J"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   204
      by (simp add: JS \<open>\<forall>I\<in>S. x \<in> I\<close> \<open>\<forall>I\<in>S. y \<in> I\<close>) }
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   205
  moreover
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   206
    have "\<zero> \<in> J" if "J \<in> S" for J
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   207
      by (simp add: that Sideals additive_subgroup.zero_closed ideal.axioms(1)) 
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   208
  moreover
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   209
  { fix x J
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   210
    assume "\<forall>I\<in>S. x \<in> I" and JS: "J \<in> S"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   211
    interpret ideal J R by (rule Sideals[OF JS])
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   212
    have "\<ominus> x \<in> J"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   213
      by (simp add: JS \<open>\<forall>I\<in>S. x \<in> I\<close>) }
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   214
  moreover
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   215
  { fix x y J
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   216
    assume "\<forall>I\<in>S. x \<in> I" and ycarr: "y \<in> carrier R" and JS: "J \<in> S"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   217
    interpret ideal J R by (rule Sideals[OF JS])
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   218
    have "y \<otimes> x \<in> J" "x \<otimes> y \<in> J" 
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   219
      using I_l_closed I_r_closed JS \<open>\<forall>I\<in>S. x \<in> I\<close> ycarr by blast+ }
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   220
  moreover
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   221
  { fix x
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   222
    assume "\<forall>I\<in>S. x \<in> I"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   223
    obtain I0 where I0S: "I0 \<in> S"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   224
      using notempty by blast
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   225
    interpret ideal I0 R by (rule Sideals[OF I0S])
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   226
    have "x \<in> I0"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   227
      by (simp add: I0S \<open>\<forall>I\<in>S. x \<in> I\<close>) 
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   228
    with a_subset have "x \<in> carrier R" by fast }
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   229
  ultimately show ?thesis
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   230
    by unfold_locales (auto simp: Inter_eq simp flip: a_inv_def)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   231
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   232
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   233
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   234
subsection \<open>Addition of Ideals\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   235
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   236
lemma (in ring) add_ideals:
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   237
  assumes idealI: "ideal I R" and idealJ: "ideal J R"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   238
  shows "ideal (I <+> J) R"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   239
proof (rule ideal.intro)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   240
  show "additive_subgroup (I <+> J) R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   241
    by (intro ideal.axioms[OF idealI] ideal.axioms[OF idealJ] add_additive_subgroups)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   242
  show "ring R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   243
    by (rule is_ring)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   244
  show "ideal_axioms (I <+> J) R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   245
  proof -
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   246
    { fix x i j
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   247
      assume xcarr: "x \<in> carrier R" and iI: "i \<in> I" and jJ: "j \<in> J"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   248
      from xcarr ideal.Icarr[OF idealI iI] ideal.Icarr[OF idealJ jJ]
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   249
      have "\<exists>h\<in>I. \<exists>k\<in>J. (i \<oplus> j) \<otimes> x = h \<oplus> k"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   250
        by (meson iI ideal.I_r_closed idealJ jJ l_distr local.idealI) }
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   251
    moreover
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   252
    { fix x i j
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   253
      assume xcarr: "x \<in> carrier R" and iI: "i \<in> I" and jJ: "j \<in> J"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   254
      from xcarr ideal.Icarr[OF idealI iI] ideal.Icarr[OF idealJ jJ]
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   255
      have "\<exists>h\<in>I. \<exists>k\<in>J. x \<otimes> (i \<oplus> j) = h \<oplus> k"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   256
        by (meson iI ideal.I_l_closed idealJ jJ local.idealI r_distr) }
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   257
    ultimately show "ideal_axioms (I <+> J) R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   258
      by (intro ideal_axioms.intro) (auto simp: set_add_defs)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   259
  qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   260
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   261
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   262
subsection (in ring) \<open>Ideals generated by a subset of @{term "carrier R"}\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   263
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   264
text \<open>@{term genideal} generates an ideal\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   265
lemma (in ring) genideal_ideal:
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   266
  assumes Scarr: "S \<subseteq> carrier R"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   267
  shows "ideal (Idl S) R"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   268
unfolding genideal_def
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   269
proof (rule i_Intersect, fast, simp)
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   270
  from oneideal and Scarr
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   271
  show "\<exists>I. ideal I R \<and> S \<le> I" by fast
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   272
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   273
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   274
lemma (in ring) genideal_self:
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   275
  assumes "S \<subseteq> carrier R"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   276
  shows "S \<subseteq> Idl S"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   277
  unfolding genideal_def by fast
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   278
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   279
lemma (in ring) genideal_self':
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   280
  assumes carr: "i \<in> carrier R"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   281
  shows "i \<in> Idl {i}"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   282
  by (simp add: genideal_def)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   283
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   284
text \<open>@{term genideal} generates the minimal ideal\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   285
lemma (in ring) genideal_minimal:
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   286
  assumes "ideal I R" "S \<subseteq> I"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   287
  shows "Idl S \<subseteq> I"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   288
  unfolding genideal_def by rule (elim InterD, simp add: assms)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   289
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   290
text \<open>Generated ideals and subsets\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   291
lemma (in ring) Idl_subset_ideal:
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   292
  assumes Iideal: "ideal I R"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   293
    and Hcarr: "H \<subseteq> carrier R"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   294
  shows "(Idl H \<subseteq> I) = (H \<subseteq> I)"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   295
proof
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   296
  assume a: "Idl H \<subseteq> I"
23350
50c5b0912a0c tuned proofs: avoid implicit prems;
wenzelm
parents: 20318
diff changeset
   297
  from Hcarr have "H \<subseteq> Idl H" by (rule genideal_self)
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   298
  with a show "H \<subseteq> I" by simp
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   299
next
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   300
  fix x
47409
c5be1120980d tuned proofs;
wenzelm
parents: 44677
diff changeset
   301
  assume "H \<subseteq> I"
c5be1120980d tuned proofs;
wenzelm
parents: 44677
diff changeset
   302
  with Iideal have "I \<in> {I. ideal I R \<and> H \<subseteq> I}" by fast
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   303
  then show "Idl H \<subseteq> I" unfolding genideal_def by fast
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   304
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   305
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   306
lemma (in ring) subset_Idl_subset:
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   307
  assumes Icarr: "I \<subseteq> carrier R"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   308
    and HI: "H \<subseteq> I"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   309
  shows "Idl H \<subseteq> Idl I"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   310
proof -
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   311
  from Icarr have Iideal: "ideal (Idl I) R"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   312
    by (rule genideal_ideal)
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   313
  from HI and Icarr have "H \<subseteq> carrier R"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   314
    by fast
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   315
  with Iideal have "(H \<subseteq> Idl I) = (Idl H \<subseteq> Idl I)"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   316
    by (rule Idl_subset_ideal[symmetric])
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   317
  then show "Idl H \<subseteq> Idl I"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   318
    by (meson HI Icarr genideal_self order_trans)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   319
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   320
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   321
lemma (in ring) Idl_subset_ideal':
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   322
  assumes acarr: "a \<in> carrier R" and bcarr: "b \<in> carrier R"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   323
  shows "Idl {a} \<subseteq> Idl {b} \<longleftrightarrow> a \<in> Idl {b}"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   324
proof -
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   325
  have "Idl {a} \<subseteq> Idl {b} \<longleftrightarrow> {a} \<subseteq> Idl {b}"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   326
    by (simp add: Idl_subset_ideal acarr bcarr genideal_ideal)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   327
  also have "\<dots> \<longleftrightarrow> a \<in> Idl {b}"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   328
    by blast
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   329
  finally show ?thesis .
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   330
qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   331
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   332
lemma (in ring) genideal_zero: "Idl {\<zero>} = {\<zero>}"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   333
proof
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   334
  show "Idl {\<zero>} \<subseteq> {\<zero>}"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   335
    by (simp add: genideal_minimal zeroideal)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   336
  show "{\<zero>} \<subseteq> Idl {\<zero>}"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   337
    by (simp add: genideal_self')
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   338
qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   339
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   340
lemma (in ring) genideal_one: "Idl {\<one>} = carrier R"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   341
proof -
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   342
  interpret ideal "Idl {\<one>}" "R" by (rule genideal_ideal) fast
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   343
  show "Idl {\<one>} = carrier R"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   344
    using genideal_self' one_imp_carrier by blast
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   345
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   346
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   347
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   348
text \<open>Generation of Principal Ideals in Commutative Rings\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   349
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   350
definition cgenideal :: "_ \<Rightarrow> 'a \<Rightarrow> 'a set"  ("PIdl\<index> _" [80] 79)
68604
57721285d4ef elimination of some "smt"
paulson <lp15@cam.ac.uk>
parents: 68464
diff changeset
   351
  where "cgenideal R a \<equiv> {x \<otimes>\<^bsub>R\<^esub> a | x. x \<in> carrier R}"
57721285d4ef elimination of some "smt"
paulson <lp15@cam.ac.uk>
parents: 68464
diff changeset
   352
57721285d4ef elimination of some "smt"
paulson <lp15@cam.ac.uk>
parents: 68464
diff changeset
   353
lemma cginideal_def': "cgenideal R a = (\<lambda>x. x \<otimes>\<^bsub>R\<^esub> a) ` carrier R"
57721285d4ef elimination of some "smt"
paulson <lp15@cam.ac.uk>
parents: 68464
diff changeset
   354
  by (auto simp add: cgenideal_def)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   355
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   356
text \<open>genhideal (?) really generates an ideal\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   357
lemma (in cring) cgenideal_ideal:
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   358
  assumes acarr: "a \<in> carrier R"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   359
  shows "ideal (PIdl a) R"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   360
  unfolding cgenideal_def
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   361
proof (intro subgroup.intro idealI[OF is_ring], simp_all)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   362
  show "{x \<otimes> a |x. x \<in> carrier R} \<subseteq> carrier R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   363
    by (blast intro: acarr)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   364
  show "\<And>x y. \<lbrakk>\<exists>u. x = u \<otimes> a \<and> u \<in> carrier R; \<exists>x. y = x \<otimes> a \<and> x \<in> carrier R\<rbrakk>
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   365
              \<Longrightarrow> \<exists>v. x \<oplus> y = v \<otimes> a \<and> v \<in> carrier R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   366
    by (metis assms cring.cring_simprules(1) is_cring l_distr)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   367
  show "\<exists>x. \<zero> = x \<otimes> a \<and> x \<in> carrier R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   368
    by (metis assms l_null zero_closed)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   369
  show "\<And>x. \<exists>u. x = u \<otimes> a \<and> u \<in> carrier R 
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   370
            \<Longrightarrow> \<exists>v. inv\<^bsub>add_monoid R\<^esub> x = v \<otimes> a \<and> v \<in> carrier R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   371
    by (metis a_inv_def add.inv_closed assms l_minus)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   372
  show "\<And>b x. \<lbrakk>\<exists>x. b = x \<otimes> a \<and> x \<in> carrier R; x \<in> carrier R\<rbrakk>
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   373
       \<Longrightarrow> \<exists>z. x \<otimes> b = z \<otimes> a \<and> z \<in> carrier R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   374
    by (metis assms m_assoc m_closed)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   375
  show "\<And>b x. \<lbrakk>\<exists>x. b = x \<otimes> a \<and> x \<in> carrier R; x \<in> carrier R\<rbrakk>
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   376
       \<Longrightarrow> \<exists>z. b \<otimes> x = z \<otimes> a \<and> z \<in> carrier R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   377
    by (metis assms m_assoc m_comm m_closed)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   378
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   379
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   380
lemma (in ring) cgenideal_self:
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   381
  assumes icarr: "i \<in> carrier R"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   382
  shows "i \<in> PIdl i"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   383
  unfolding cgenideal_def
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   384
proof simp
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   385
  from icarr have "i = \<one> \<otimes> i"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   386
    by simp
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   387
  with icarr show "\<exists>x. i = x \<otimes> i \<and> x \<in> carrier R"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   388
    by fast
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   389
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   390
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   391
text \<open>@{const "cgenideal"} is minimal\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   392
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   393
lemma (in ring) cgenideal_minimal:
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   394
  assumes "ideal J R"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   395
  assumes aJ: "a \<in> J"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   396
  shows "PIdl a \<subseteq> J"
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   397
proof -
29240
bb81c3709fb6 More porting to new locales.
ballarin
parents: 29237
diff changeset
   398
  interpret ideal J R by fact
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   399
  show ?thesis
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   400
    unfolding cgenideal_def
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   401
    using I_l_closed aJ by blast
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   402
qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   403
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   404
lemma (in cring) cgenideal_eq_genideal:
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   405
  assumes icarr: "i \<in> carrier R"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   406
  shows "PIdl i = Idl {i}"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   407
proof
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   408
  show "PIdl i \<subseteq> Idl {i}"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   409
    by (simp add: cgenideal_minimal genideal_ideal genideal_self' icarr)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   410
  show "Idl {i} \<subseteq> PIdl i"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   411
    by (simp add: cgenideal_ideal cgenideal_self genideal_minimal icarr)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   412
qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   413
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   414
lemma (in cring) cgenideal_eq_rcos: "PIdl i = carrier R #> i"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   415
  unfolding cgenideal_def r_coset_def by fast
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   416
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   417
lemma (in cring) cgenideal_is_principalideal:
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   418
  assumes "i \<in> carrier R"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   419
  shows "principalideal (PIdl i) R"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   420
proof -
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   421
  have "\<exists>i'\<in>carrier R. PIdl i = Idl {i'}"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   422
    using cgenideal_eq_genideal assms by auto
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   423
  then show ?thesis
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   424
    by (simp add: cgenideal_ideal assms principalidealI)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   425
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   426
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   427
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   428
subsection \<open>Union of Ideals\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   429
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   430
lemma (in ring) union_genideal:
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   431
  assumes idealI: "ideal I R" and idealJ: "ideal J R"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   432
  shows "Idl (I \<union> J) = I <+> J"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   433
proof
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   434
  show "Idl (I \<union> J) \<subseteq> I <+> J"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   435
  proof (rule ring.genideal_minimal [OF is_ring])
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   436
    show "ideal (I <+> J) R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   437
      by (rule add_ideals[OF idealI idealJ])
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   438
    have "\<And>x. x \<in> I \<Longrightarrow> \<exists>xa\<in>I. \<exists>xb\<in>J. x = xa \<oplus> xb"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   439
      by (metis additive_subgroup.zero_closed ideal.Icarr idealJ ideal_def local.idealI r_zero)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   440
    moreover have "\<And>x. x \<in> J \<Longrightarrow> \<exists>xa\<in>I. \<exists>xb\<in>J. x = xa \<oplus> xb"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   441
      by (metis additive_subgroup.zero_closed ideal.Icarr idealJ ideal_def l_zero local.idealI)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   442
    ultimately show "I \<union> J \<subseteq> I <+> J"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   443
      by (auto simp: set_add_defs) 
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   444
  qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   445
next
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   446
  show "I <+> J \<subseteq> Idl (I \<union> J)"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   447
    by (auto simp: set_add_defs genideal_def additive_subgroup.a_closed ideal_def set_mp)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   448
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   449
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   450
subsection \<open>Properties of Principal Ideals\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   451
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   452
text \<open>The zero ideal is a principal ideal\<close>
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   453
corollary (in ring) zeropideal: "principalideal {\<zero>} R"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   454
  using genideal_zero principalidealI zeroideal by blast
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   455
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   456
text \<open>The unit ideal is a principal ideal\<close>
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   457
corollary (in ring) onepideal: "principalideal (carrier R) R"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   458
  using genideal_one oneideal principalidealI by blast
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   459
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   460
text \<open>Every principal ideal is a right coset of the carrier\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   461
lemma (in principalideal) rcos_generate:
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   462
  assumes "cring R"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   463
  shows "\<exists>x\<in>I. I = carrier R #> x"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   464
proof -
29237
e90d9d51106b More porting to new locales.
ballarin
parents: 27717
diff changeset
   465
  interpret cring R by fact
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   466
  from generate obtain i where icarr: "i \<in> carrier R" and I1: "I = Idl {i}"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   467
    by fast+
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   468
  then have "I = PIdl i"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   469
    by (simp add: cgenideal_eq_genideal)
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   470
  moreover have "i \<in> I"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   471
    by (simp add: I1 genideal_self' icarr)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   472
  moreover have "PIdl i = carrier R #> i"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   473
    unfolding cgenideal_def r_coset_def by fast
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   474
  ultimately show "\<exists>x\<in>I. I = carrier R #> x"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   475
    by fast
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   476
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   477
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   478
68445
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   479
(* Next lemma contributed by Paulo Emílio de Vilhena. *)
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   480
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   481
text \<open>This next lemma would be trivial if placed in a theory that imports QuotRing,
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   482
      but it makes more sense to have it here (easier to find and coherent with the
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   483
      previous developments).\<close>
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   484
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   485
lemma (in cring) cgenideal_prod:
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   486
  assumes "a \<in> carrier R" "b \<in> carrier R"
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   487
  shows "(PIdl a) <#> (PIdl b) = PIdl (a \<otimes> b)"
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   488
proof -
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   489
  have "(carrier R #> a) <#> (carrier R #> b) = carrier R #> (a \<otimes> b)"
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   490
  proof
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   491
    show "(carrier R #> a) <#> (carrier R #> b) \<subseteq> carrier R #> a \<otimes> b"
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   492
    proof
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   493
      fix x assume "x \<in> (carrier R #> a) <#> (carrier R #> b)"
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   494
      then obtain r1 r2 where r1: "r1 \<in> carrier R" and r2: "r2 \<in> carrier R"
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   495
                          and "x = (r1 \<otimes> a) \<otimes> (r2 \<otimes> b)"
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   496
        unfolding set_mult_def r_coset_def by blast
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   497
      hence "x = (r1 \<otimes> r2) \<otimes> (a \<otimes> b)"
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   498
        by (simp add: assms local.ring_axioms m_lcomm ring.ring_simprules(11))
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   499
      thus "x \<in> carrier R #> a \<otimes> b"
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   500
        unfolding r_coset_def using r1 r2 assms by blast 
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   501
    qed
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   502
  next
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   503
    show "carrier R #> a \<otimes> b \<subseteq> (carrier R #> a) <#> (carrier R #> b)"
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   504
    proof
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   505
      fix x assume "x \<in> carrier R #> a \<otimes> b"
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   506
      then obtain r where r: "r \<in> carrier R" "x = r \<otimes> (a \<otimes> b)"
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   507
        unfolding r_coset_def by blast
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   508
      hence "x = (r \<otimes> a) \<otimes> (\<one> \<otimes> b)"
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   509
        using assms by (simp add: m_assoc)
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   510
      thus "x \<in> (carrier R #> a) <#> (carrier R #> b)"
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   511
        unfolding set_mult_def r_coset_def using assms r by blast
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   512
    qed
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   513
  qed
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   514
  thus ?thesis
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   515
    using cgenideal_eq_rcos[of a] cgenideal_eq_rcos[of b] cgenideal_eq_rcos[of "a \<otimes> b"] by simp
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   516
qed
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   517
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   518
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   519
subsection \<open>Prime Ideals\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   520
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   521
lemma (in ideal) primeidealCD:
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   522
  assumes "cring R"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   523
  assumes notprime: "\<not> primeideal I R"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   524
  shows "carrier R = I \<or> (\<exists>a b. a \<in> carrier R \<and> b \<in> carrier R \<and> a \<otimes> b \<in> I \<and> a \<notin> I \<and> b \<notin> I)"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   525
proof (rule ccontr, clarsimp)
29237
e90d9d51106b More porting to new locales.
ballarin
parents: 27717
diff changeset
   526
  interpret cring R by fact
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   527
  assume InR: "carrier R \<noteq> I"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   528
    and "\<forall>a. a \<in> carrier R \<longrightarrow> (\<forall>b. a \<otimes> b \<in> I \<longrightarrow> b \<in> carrier R \<longrightarrow> a \<in> I \<or> b \<in> I)"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   529
  then have I_prime: "\<And> a b. \<lbrakk>a \<in> carrier R; b \<in> carrier R; a \<otimes> b \<in> I\<rbrakk> \<Longrightarrow> a \<in> I \<or> b \<in> I"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   530
    by simp
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   531
  have "primeideal I R"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   532
    by (simp add: I_prime InR is_cring is_ideal primeidealI)
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   533
  with notprime show False by simp
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   534
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   535
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   536
lemma (in ideal) primeidealCE:
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   537
  assumes "cring R"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   538
  assumes notprime: "\<not> primeideal I R"
23383
5460951833fa tuned proofs: avoid implicit prems;
wenzelm
parents: 23350
diff changeset
   539
  obtains "carrier R = I"
5460951833fa tuned proofs: avoid implicit prems;
wenzelm
parents: 23350
diff changeset
   540
    | "\<exists>a b. a \<in> carrier R \<and> b \<in> carrier R \<and> a \<otimes> b \<in> I \<and> a \<notin> I \<and> b \<notin> I"
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   541
proof -
30729
461ee3e49ad3 interpretation/interpret: prefixes are mandatory by default;
wenzelm
parents: 30363
diff changeset
   542
  interpret R: cring R by fact
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   543
  assume "carrier R = I ==> thesis"
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   544
    and "\<exists>a b. a \<in> carrier R \<and> b \<in> carrier R \<and> a \<otimes> b \<in> I \<and> a \<notin> I \<and> b \<notin> I \<Longrightarrow> thesis"
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   545
  then show thesis using primeidealCD [OF R.is_cring notprime] by blast
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   546
qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   547
63167
0909deb8059b isabelle update_cartouches -c -t;
wenzelm
parents: 63040
diff changeset
   548
text \<open>If \<open>{\<zero>}\<close> is a prime ideal of a commutative ring, the ring is a domain\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   549
lemma (in cring) zeroprimeideal_domainI:
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   550
  assumes pi: "primeideal {\<zero>} R"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   551
  shows "domain R"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   552
proof (intro domain.intro is_cring domain_axioms.intro)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   553
  show "\<one> \<noteq> \<zero>"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   554
    using genideal_one genideal_zero pi primeideal.I_notcarr by force
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   555
  show "a = \<zero> \<or> b = \<zero>" if ab: "a \<otimes> b = \<zero>" and carr: "a \<in> carrier R" "b \<in> carrier R" for a b
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   556
  proof -
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   557
    interpret primeideal "{\<zero>}" "R" by (rule pi)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   558
    show "a = \<zero> \<or> b = \<zero>"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   559
      using I_prime ab carr by blast
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   560
  qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   561
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   562
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   563
corollary (in cring) domain_eq_zeroprimeideal: "domain R = primeideal {\<zero>} R"
68443
43055b016688 New material from Martin Baillon and Paulo Emílio de Vilhena
paulson <lp15@cam.ac.uk>
parents: 67443
diff changeset
   564
  using domain.zeroprimeideal zeroprimeideal_domainI by blast
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   565
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   566
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   567
subsection \<open>Maximal Ideals\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   568
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   569
lemma (in ideal) helper_I_closed:
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   570
  assumes carr: "a \<in> carrier R" "x \<in> carrier R" "y \<in> carrier R"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   571
    and axI: "a \<otimes> x \<in> I"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   572
  shows "a \<otimes> (x \<otimes> y) \<in> I"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   573
proof -
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   574
  from axI and carr have "(a \<otimes> x) \<otimes> y \<in> I"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   575
    by (simp add: I_r_closed)
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   576
  also from carr have "(a \<otimes> x) \<otimes> y = a \<otimes> (x \<otimes> y)"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   577
    by (simp add: m_assoc)
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   578
  finally show "a \<otimes> (x \<otimes> y) \<in> I" .
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   579
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   580
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   581
lemma (in ideal) helper_max_prime:
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   582
  assumes "cring R"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   583
  assumes acarr: "a \<in> carrier R"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   584
  shows "ideal {x\<in>carrier R. a \<otimes> x \<in> I} R"
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   585
proof -
29237
e90d9d51106b More porting to new locales.
ballarin
parents: 27717
diff changeset
   586
  interpret cring R by fact
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   587
  show ?thesis 
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   588
  proof (rule idealI, simp_all)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   589
    show "ring R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   590
      by (simp add: local.ring_axioms)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   591
    show "subgroup {x \<in> carrier R. a \<otimes> x \<in> I} (add_monoid R)"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   592
      by (rule subgroup.intro) (auto simp: r_distr acarr r_minus simp flip: a_inv_def)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   593
    show "\<And>b x. \<lbrakk>b \<in> carrier R \<and> a \<otimes> b \<in> I; x \<in> carrier R\<rbrakk>
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   594
                 \<Longrightarrow> a \<otimes> (x \<otimes> b) \<in> I"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   595
      using acarr helper_I_closed m_comm by auto
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   596
    show "\<And>b x. \<lbrakk>b \<in> carrier R \<and> a \<otimes> b \<in> I; x \<in> carrier R\<rbrakk>
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   597
                \<Longrightarrow> a \<otimes> (b \<otimes> x) \<in> I"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   598
      by (simp add: acarr helper_I_closed)
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   599
  qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   600
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   601
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   602
text \<open>In a cring every maximal ideal is prime\<close>
63633
2accfb71e33b is_prime -> prime
eberlm <eberlm@in.tum.de>
parents: 63167
diff changeset
   603
lemma (in cring) maximalideal_prime:
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   604
  assumes "maximalideal I R"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   605
  shows "primeideal I R"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   606
proof -
29237
e90d9d51106b More porting to new locales.
ballarin
parents: 27717
diff changeset
   607
  interpret maximalideal I R by fact
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   608
  show ?thesis 
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   609
  proof (rule ccontr)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   610
    assume neg: "\<not> primeideal I R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   611
    then obtain a b where acarr: "a \<in> carrier R" and bcarr: "b \<in> carrier R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   612
      and abI: "a \<otimes> b \<in> I" and anI: "a \<notin> I" and bnI: "b \<notin> I" 
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   613
      using primeidealCE [OF is_cring]
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   614
      by (metis I_notcarr)
63040
eb4ddd18d635 eliminated old 'def';
wenzelm
parents: 61952
diff changeset
   615
    define J where "J = {x\<in>carrier R. a \<otimes> x \<in> I}"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   616
    from is_cring and acarr have idealJ: "ideal J R"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   617
      unfolding J_def by (rule helper_max_prime)
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   618
    have IsubJ: "I \<subseteq> J"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   619
      using I_l_closed J_def a_Hcarr acarr by blast
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   620
    from abI and acarr bcarr have "b \<in> J"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   621
      unfolding J_def by fast
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   622
    with bnI have JnI: "J \<noteq> I" by fast
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   623
    have "\<one> \<notin> J"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   624
      unfolding J_def by (simp add: acarr anI)
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   625
    then have Jncarr: "J \<noteq> carrier R" by fast
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   626
    interpret ideal J R by (rule idealJ)    
27611
2c01c0bdb385 Removed uses of context element includes.
ballarin
parents: 26203
diff changeset
   627
    have "J = I \<or> J = carrier R"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   628
      by (simp add: I_maximal IsubJ a_subset is_ideal)
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   629
    with JnI and Jncarr show False by simp
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   630
  qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   631
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   632
35849
b5522b51cb1e standard headers;
wenzelm
parents: 35848
diff changeset
   633
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   634
subsection \<open>Derived Theorems\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   635
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   636
text \<open>A non-zero cring that has only the two trivial ideals is a field\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   637
lemma (in cring) trivialideals_fieldI:
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   638
  assumes carrnzero: "carrier R \<noteq> {\<zero>}"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   639
    and haveideals: "{I. ideal I R} = {{\<zero>}, carrier R}"
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   640
  shows "field R"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   641
proof (intro cring_fieldI equalityI)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   642
  show "Units R \<subseteq> carrier R - {\<zero>}"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   643
    by (metis Diff_empty Units_closed Units_r_inv_ex carrnzero l_null one_zeroD subsetI subset_Diff_insert)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   644
  show "carrier R - {\<zero>} \<subseteq> Units R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   645
  proof
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   646
    fix x
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   647
    assume xcarr': "x \<in> carrier R - {\<zero>}"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   648
    then have xcarr: "x \<in> carrier R" and xnZ: "x \<noteq> \<zero>" by auto
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   649
    from xcarr have xIdl: "ideal (PIdl x) R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   650
      by (intro cgenideal_ideal) fast
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   651
    have "PIdl x \<noteq> {\<zero>}"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   652
      using xcarr xnZ cgenideal_self by blast 
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   653
    with haveideals have "PIdl x = carrier R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   654
      by (blast intro!: xIdl)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   655
    then have "\<one> \<in> PIdl x" by simp
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   656
    then have "\<exists>y. \<one> = y \<otimes> x \<and> y \<in> carrier R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   657
      unfolding cgenideal_def by blast
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   658
    then obtain y where ycarr: " y \<in> carrier R" and ylinv: "\<one> = y \<otimes> x"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   659
      by fast    
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   660
    have "\<exists>y \<in> carrier R. y \<otimes> x = \<one> \<and> x \<otimes> y = \<one>"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   661
      using m_comm xcarr ycarr ylinv by auto
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   662
    with xcarr show "x \<in> Units R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   663
      unfolding Units_def by fast
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   664
  qed
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   665
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   666
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   667
lemma (in field) all_ideals: "{I. ideal I R} = {{\<zero>}, carrier R}"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   668
proof (intro equalityI subsetI)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   669
  fix I
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   670
  assume a: "I \<in> {I. ideal I R}"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   671
  then interpret ideal I R by simp
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   672
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   673
  show "I \<in> {{\<zero>}, carrier R}"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   674
  proof (cases "\<exists>a. a \<in> I - {\<zero>}")
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   675
    case True
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   676
    then obtain a where aI: "a \<in> I" and anZ: "a \<noteq> \<zero>"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   677
      by fast+
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   678
    have aUnit: "a \<in> Units R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   679
      by (simp add: aI anZ field_Units)
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   680
    then have a: "a \<otimes> inv a = \<one>" by (rule Units_r_inv)
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   681
    from aI and aUnit have "a \<otimes> inv a \<in> I"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   682
      by (simp add: I_r_closed del: Units_r_inv)
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   683
    then have oneI: "\<one> \<in> I" by (simp add: a[symmetric])
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   684
    have "carrier R \<subseteq> I"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   685
      using oneI one_imp_carrier by auto
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   686
    with a_subset have "I = carrier R" by fast
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   687
    then show "I \<in> {{\<zero>}, carrier R}" by fast
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   688
  next
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   689
    case False
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   690
    then have IZ: "\<And>a. a \<in> I \<Longrightarrow> a = \<zero>" by simp
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   691
    have a: "I \<subseteq> {\<zero>}"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   692
      using False by auto
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   693
    have "\<zero> \<in> I" by simp
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   694
    with a have "I = {\<zero>}" by fast
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   695
    then show "I \<in> {{\<zero>}, carrier R}" by fast
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   696
  qed
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   697
qed (auto simp: zeroideal oneideal)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   698
68445
c183a6a69f2d reorganisation of Algebra: new material from Baillon and Vilhena, removal of duplicate names, elimination of "More_" theories
paulson <lp15@cam.ac.uk>
parents: 68443
diff changeset
   699
\<comment>\<open>"Jacobson Theorem 2.2"\<close>
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   700
lemma (in cring) trivialideals_eq_field:
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   701
  assumes carrnzero: "carrier R \<noteq> {\<zero>}"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   702
  shows "({I. ideal I R} = {{\<zero>}, carrier R}) = field R"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   703
  by (fast intro!: trivialideals_fieldI[OF carrnzero] field.all_ideals)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   704
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   705
61382
efac889fccbc isabelle update_cartouches;
wenzelm
parents: 47409
diff changeset
   706
text \<open>Like zeroprimeideal for domains\<close>
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   707
lemma (in field) zeromaximalideal: "maximalideal {\<zero>} R"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   708
proof (intro maximalidealI zeroideal)
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   709
  from one_not_zero have "\<one> \<notin> {\<zero>}" by simp
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   710
  with one_closed show "carrier R \<noteq> {\<zero>}" by fast
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   711
next
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   712
  fix J
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   713
  assume Jideal: "ideal J R"
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   714
  then have "J \<in> {I. ideal I R}" by fast
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   715
  with all_ideals show "J = {\<zero>} \<or> J = carrier R"
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   716
    by simp
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   717
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   718
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   719
lemma (in cring) zeromaximalideal_fieldI:
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   720
  assumes zeromax: "maximalideal {\<zero>} R"
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   721
  shows "field R"
68464
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   722
proof (intro trivialideals_fieldI maximalideal.I_notcarr[OF zeromax])
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   723
  have "J = carrier R" if Jn0: "J \<noteq> {\<zero>}" and idealJ: "ideal J R" for J
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   724
  proof -
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   725
    interpret ideal J R by (rule idealJ)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   726
    have "{\<zero>} \<subseteq> J"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   727
      by force
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   728
    from zeromax idealJ this a_subset
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   729
    have "J = {\<zero>} \<or> J = carrier R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   730
      by (rule maximalideal.I_maximal)
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   731
    with Jn0 show "J = carrier R"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   732
      by simp
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   733
  qed
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   734
  then show "{I. ideal I R} = {{\<zero>}, carrier R}"
3ead36cbe6b7 De-applied Ideal.thy
paulson <lp15@cam.ac.uk>
parents: 68458
diff changeset
   735
    by (auto simp: zeroideal oneideal)
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   736
qed
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   737
44677
3fb27b19e058 misc tuning and simplification of proofs;
wenzelm
parents: 44106
diff changeset
   738
lemma (in cring) zeromaximalideal_eq_field: "maximalideal {\<zero>} R = field R"
68443
43055b016688 New material from Martin Baillon and Paulo Emílio de Vilhena
paulson <lp15@cam.ac.uk>
parents: 67443
diff changeset
   739
  using field.zeromaximalideal zeromaximalideal_fieldI by blast
20318
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   740
0e0ea63fe768 Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
diff changeset
   741
end