Commit 2023-12-23 10:52 ea70e843
View on Github →refactor: Deduplicate monotonicity of •
lemmas (#9179)
Remove the duplicates introduced in #8869 by sorting the lemmas in Algebra.Order.SMul
into three files:
Algebra.Order.Module.Defs
for the order isomorphism induced by scalar multiplication by a positivity elementAlgebra.Order.Module.Pointwise
for the order properties of scalar multiplication of sets. This file is new. I credit myself for https://github.com/leanprover-community/mathlib/pull/9078Algebra.Order.Module.OrderedSMul
: The material aboutOrderedSMul
per se. Inherits the copyright header fromAlgebra.Order.SMul
. This file should eventually be deleted. I move each#align
to the correct file. On top of that, I delete unused redundantOrderedSMul
instances (they were useful in Lean 3, but not anymore) andeq_of_smul_eq_smul_of_pos_of_le
/eq_of_smul_eq_smul_of_neg_of_le
since those lemmas are weird and unused.