Skip to content

Commit

Permalink
lint
Browse files Browse the repository at this point in the history
  • Loading branch information
collares committed Oct 22, 2023
1 parent b0bc32e commit 8f501cb
Showing 1 changed file with 3 additions and 4 deletions.
7 changes: 3 additions & 4 deletions Mathlib/Data/Real/ENNReal.lean
Original file line number Diff line number Diff line change
Expand Up @@ -633,11 +633,10 @@ theorem mul_lt_top_iff {a b : ℝ≥0∞} : a * b < ∞ ↔ a < ∞ ∧ b < ∞
rw [← or_assoc, or_iff_not_imp_right, or_iff_not_imp_right]
intro hb ha
exact ⟨lt_top_of_mul_ne_top_left h.ne hb, lt_top_of_mul_ne_top_right h.ne ha⟩
· have : 0 < (⊤ : ℝ≥0∞) := by decide
rintro (⟨ha, hb⟩ | rfl | rfl)
· rintro (⟨ha, hb⟩ | rfl | rfl)
· exact mul_lt_top ha.ne hb.ne
· simp [this]
· simp [this]
· simp
· simp
#align ennreal.mul_lt_top_iff ENNReal.mul_lt_top_iff

theorem mul_self_lt_top_iff {a : ℝ≥0∞} : a * a < ⊤ ↔ a < ⊤ := by
Expand Down

0 comments on commit 8f501cb

Please sign in to comment.