Skip to content

Commit

Permalink
feat: PosSMulMono ℚ α → PosSMulMono ℚ≥0 α (#17217)
Browse files Browse the repository at this point in the history
From LeanAPAP
  • Loading branch information
YaelDillies committed Oct 17, 2024
1 parent 8306205 commit 090e243
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions Mathlib/Algebra/Order/Module/Rat.lean
Original file line number Diff line number Diff line change
Expand Up @@ -12,6 +12,12 @@ import Mathlib.Data.Rat.Cast.Order

variable {α : Type*}

instance PosSMulMono.nnrat_of_rat [Preorder α] [MulAction ℚ α] [PosSMulMono ℚ α] :
PosSMulMono ℚ≥0 α where elim _q hq _a₁ _a₂ ha := smul_le_smul_of_nonneg_left (α := ℚ) ha hq

instance PosSMulStrictMono.nnrat_of_rat [Preorder α] [MulAction ℚ α] [PosSMulStrictMono ℚ α] :
PosSMulStrictMono ℚ≥0 α where elim _q hq _a₁ _a₂ ha := smul_lt_smul_of_pos_left (α := ℚ) ha hq

section LinearOrderedAddCommGroup
variable [LinearOrderedAddCommGroup α]

Expand Down

0 comments on commit 090e243

Please sign in to comment.