Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 74373b8

Browse files
committed
feat(algebra/lattice_ordered_group): add basic theory of lattice ordered groups (#8673)
Co-authored-by: Christopher Hoskin <mans0954@users.noreply.github.com>
1 parent c563692 commit 74373b8

File tree

12 files changed

+656
-16
lines changed

12 files changed

+656
-16
lines changed

docs/references.bib

Lines changed: 57 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -80,6 +80,13 @@ @Book{ axler2015
8080
publisher = {Springer}
8181
}
8282

83+
@Manual{ banasiak,
84+
author = {Banasiak},
85+
title = {Banach Lattices in Applications},
86+
organization = {University of Pretoria},
87+
address = {Pretoria, South Africa}
88+
}
89+
8390
@Book{ beals2004,
8491
author = {Richard Beals},
8592
title = {Analysis. An introduction},
@@ -137,6 +144,22 @@ @Book{ billingsley1999
137144
url = {https://doi.org/10.1002/9780470316962}
138145
}
139146

147+
@Article{ birkhoff1942,
148+
author = {Birkhoff, Garrett},
149+
title = {Lattice, ordered groups},
150+
journal = {Ann. of Math. (2)},
151+
fjournal = {Annals of Mathematics. Second Series},
152+
volume = {43},
153+
year = {1942},
154+
pages = {298--331},
155+
issn = {0003-486X},
156+
mrclass = {20.0X},
157+
mrnumber = {6550},
158+
mrreviewer = {H. Wallman},
159+
doi = {10.2307/1968871},
160+
url = {https://doi.org/10.2307/1968871}
161+
}
162+
140163
@Book{ borceux-vol1,
141164
title = {Handbook of Categorical Algebra: Volume 1, Basic Category
142165
Theory},
@@ -210,6 +233,19 @@ @Book{ bourbaki1975b
210233
mrnumber = {2109105}
211234
}
212235

236+
@Book{ bourbaki1981,
237+
author = {Bourbaki, N.},
238+
title = {Algebra. {II}. {C}hapters 4--7},
239+
series = {Elements of Mathematics (Berlin)},
240+
note = {Translated from the French by P. M. Cohn and J. Howie},
241+
publisher = {Springer-Verlag, Berlin},
242+
year = {1990},
243+
pages = {vii+461},
244+
isbn = {3-540-19375-8},
245+
mrclass = {00A05 (12-01 13-01)},
246+
mrnumber = {1080964}
247+
}
248+
213249
@Article{ cadiou1972,
214250
title = {Recursive definitions of partial functions and their
215251
computations},
@@ -432,6 +468,19 @@ @InProceedings{ flypitch_itp
432468
continuum hypothesis, Boolean-valued models, Lean}
433469
}
434470

471+
@Book{ fuchs1963,
472+
author = {Fuchs, L.},
473+
title = {Partially ordered algebraic systems},
474+
publisher = {Pergamon Press, Oxford-London-New York-Paris;
475+
Addison-Wesley Publishing Co., Inc., Reading, Mass.-Palo
476+
Alto, Calif.-London},
477+
year = {1963},
478+
pages = {ix+229},
479+
mrclass = {06.00 (20.00)},
480+
mrnumber = {0171864},
481+
mrreviewer = {P. F. Conrad}
482+
}
483+
435484
@InProceedings{ fuerer-lochbihler-schneider-traytel2020,
436485
author = {Basil F{\"{u}}rer and Andreas Lochbihler and Joshua
437486
Schneider and Dmitriy Traytel},
@@ -1190,6 +1239,14 @@ @Misc{ wedhorn_adic
11901239
eprint = {arXiv:1910.05934}
11911240
}
11921241

1242+
@TechReport{ zaanen1966,
1243+
author = {Zaanen, A. C.},
1244+
title = {Lectures on "Riesz Spaces"},
1245+
institution = {Euratom},
1246+
year = {1966},
1247+
number = {EUR 3140.e}
1248+
}
1249+
11931250
@Article{ zbMATH06785026,
11941251
author = {John F. {Clauser} and Michael A. {Horne} and Abner
11951252
{Shimony} and Richard A. {Holt}},

src/algebra/field_power.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -159,7 +159,7 @@ lemma fpow_even_abs (a : K) {p : ℤ} (hp : even p) :
159159
abs a ^ p = a ^ p :=
160160
begin
161161
cases le_or_lt a (-a) with h h;
162-
simp [abs, h, max_eq_left_of_lt, fpow_even_neg _ hp]
162+
simp [abs_eq_max_neg, h, max_eq_left_of_lt, fpow_even_neg _ hp]
163163
end
164164

165165
@[simp] lemma fpow_bit0_abs (a : K) (p : ℤ) :

src/algebra/group/basic.lean

Lines changed: 5 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -451,6 +451,11 @@ by rw [mul_inv_rev, mul_comm]
451451
lemma div_eq_of_eq_mul' {a b c : G} (h : a = b * c) : a / b = c :=
452452
by rw [h, div_eq_mul_inv, mul_comm, inv_mul_cancel_left]
453453

454+
@[to_additive]
455+
lemma div_mul_comm (a b c d : G) : a / b * (c / d) = a * c / (b * d) :=
456+
by rw [div_eq_mul_inv, div_eq_mul_inv, div_eq_mul_inv, mul_inv_rev, mul_assoc, mul_assoc,
457+
mul_left_cancel_iff, mul_comm, mul_assoc]
458+
454459
end comm_group
455460

456461
section add_comm_group

0 commit comments

Comments
 (0)