# HG changeset patch # User ballarin # Date 1504208881 -7200 # Node ID 2db3fe23fdaff76cfafc7d59d9a1c1eb03936f16 # Parent 6a034c6c423fa2553d57d413d8f069eee2a0e8fe Revert 5a42eddc11c1. diff -r 6a034c6c423f -r 2db3fe23fdaf src/HOL/Algebra/Complete_Lattice.thy --- a/src/HOL/Algebra/Complete_Lattice.thy Thu Aug 31 20:19:55 2017 +0200 +++ b/src/HOL/Algebra/Complete_Lattice.thy Thu Aug 31 21:48:01 2017 +0200 @@ -7,7 +7,7 @@ *) theory Complete_Lattice -imports Lattice Group +imports Lattice begin section \Complete Lattices\ @@ -1192,43 +1192,8 @@ then show "EX i. greatest ?L i (Lower ?L B)" .. qed -theorem (in group) subgroups_complete_lattice: - "complete_lattice \carrier = {H. subgroup H G}, eq = op =, le = op \\" - (is "complete_lattice ?L") -proof (rule partial_order.complete_lattice_criterion1) - show "partial_order ?L" by (rule subgroups_partial_order) -next - have "greatest ?L (carrier G) (carrier ?L)" - by (unfold greatest_def) (simp add: subgroup.subset subgroup_self) - then show "\G. greatest ?L G (carrier ?L)" .. -next - fix A - assume L: "A \ carrier ?L" and non_empty: "A ~= {}" - then have Int_subgroup: "subgroup (\A) G" - by (fastforce intro: subgroups_Inter) - have "greatest ?L (\A) (Lower ?L A)" (is "greatest _ ?Int _") - proof (rule greatest_LowerI) - fix H - assume H: "H \ A" - with L have subgroupH: "subgroup H G" by auto - from subgroupH have groupH: "group (G \carrier := H\)" (is "group ?H") - by (rule subgroup_imp_group) - from groupH have monoidH: "monoid ?H" - by (rule group.is_monoid) - from H have Int_subset: "?Int \ H" by fastforce - then show "le ?L ?Int H" by simp - next - fix H - assume H: "H \ Lower ?L A" - with L Int_subgroup show "le ?L H ?Int" - by (fastforce simp: Lower_def intro: Inter_greatest) - next - show "A \ carrier ?L" by (rule L) - next - show "?Int \ carrier ?L" by simp (rule Int_subgroup) - qed - then show "\I. greatest ?L I (Lower ?L A)" .. -qed +text \Another example, that of the lattice of subgroups of a group, + can be found in Group theory (Section~\ref{sec:subgroup-lattice}).\ subsection \Limit preserving functions\ diff -r 6a034c6c423f -r 2db3fe23fdaf src/HOL/Algebra/Divisibility.thy --- a/src/HOL/Algebra/Divisibility.thy Thu Aug 31 20:19:55 2017 +0200 +++ b/src/HOL/Algebra/Divisibility.thy Thu Aug 31 21:48:01 2017 +0200 @@ -6,7 +6,7 @@ section \Divisibility in monoids and rings\ theory Divisibility - imports "HOL-Library.Permutation" Coset Group Lattice + imports "HOL-Library.Permutation" Coset Group begin section \Factorial Monoids\ diff -r 6a034c6c423f -r 2db3fe23fdaf src/HOL/Algebra/Group.thy --- a/src/HOL/Algebra/Group.thy Thu Aug 31 20:19:55 2017 +0200 +++ b/src/HOL/Algebra/Group.thy Thu Aug 31 21:48:01 2017 +0200 @@ -5,7 +5,7 @@ *) theory Group -imports Order "HOL-Library.FuncSet" +imports Complete_Lattice "HOL-Library.FuncSet" begin section \Monoids and Groups\ @@ -817,4 +817,42 @@ show "x \ y \ \A" by blast qed +theorem (in group) subgroups_complete_lattice: + "complete_lattice \carrier = {H. subgroup H G}, eq = op =, le = op \\" + (is "complete_lattice ?L") +proof (rule partial_order.complete_lattice_criterion1) + show "partial_order ?L" by (rule subgroups_partial_order) +next + have "greatest ?L (carrier G) (carrier ?L)" + by (unfold greatest_def) (simp add: subgroup.subset subgroup_self) + then show "\G. greatest ?L G (carrier ?L)" .. +next + fix A + assume L: "A \ carrier ?L" and non_empty: "A ~= {}" + then have Int_subgroup: "subgroup (\A) G" + by (fastforce intro: subgroups_Inter) + have "greatest ?L (\A) (Lower ?L A)" (is "greatest _ ?Int _") + proof (rule greatest_LowerI) + fix H + assume H: "H \ A" + with L have subgroupH: "subgroup H G" by auto + from subgroupH have groupH: "group (G \carrier := H\)" (is "group ?H") + by (rule subgroup_imp_group) + from groupH have monoidH: "monoid ?H" + by (rule group.is_monoid) + from H have Int_subset: "?Int \ H" by fastforce + then show "le ?L ?Int H" by simp + next + fix H + assume H: "H \ Lower ?L A" + with L Int_subgroup show "le ?L H ?Int" + by (fastforce simp: Lower_def intro: Inter_greatest) + next + show "A \ carrier ?L" by (rule L) + next + show "?Int \ carrier ?L" by simp (rule Int_subgroup) + qed + then show "\I. greatest ?L I (Lower ?L A)" .. +qed + end