Skip to content

Commit

Permalink
clenaup
Browse files Browse the repository at this point in the history
  • Loading branch information
LorenzoLuccioli committed Aug 2, 2024
1 parent 06301cf commit 1e1c0d7
Showing 1 changed file with 2 additions and 4 deletions.
6 changes: 2 additions & 4 deletions TestingLowerBounds/ForMathlib/EReal.lean
Original file line number Diff line number Diff line change
Expand Up @@ -118,8 +118,7 @@ lemma mul_ne_bot (a b : EReal) :

lemma mul_pos_iff {a b : EReal} : 0 < a * b ↔ 0 < a ∧ 0 < b ∨ a < 0 ∧ b < 0 := by
induction a, b using EReal.induction₂_symm with
| symm h =>
simp [mul_comm, h, and_comm]
| symm h => simp [mul_comm, h, and_comm]
| top_top => simp
| top_pos _ hx => simp [EReal.top_mul_coe_of_pos hx, hx]
| top_zero => simp
Expand All @@ -137,8 +136,7 @@ lemma mul_neg_iff {a b : EReal} : a * b < 0 ↔ 0 < a ∧ b < 0 ∨ a < 0 ∧ 0

lemma mul_nonneg_iff {a b : EReal} : 0 ≤ a * b ↔ 0 ≤ a ∧ 0 ≤ b ∨ a ≤ 0 ∧ b ≤ 0 := by
induction a, b using EReal.induction₂_symm with
| symm h =>
simp [mul_comm, h, and_comm]
| symm h => simp [mul_comm, h, and_comm]
| top_top => simp
| top_pos _ hx => simp [EReal.top_mul_coe_of_pos hx, hx, le_of_lt]
| top_zero => simp
Expand Down

0 comments on commit 1e1c0d7

Please sign in to comment.