Skip to content

Commit

Permalink
test linter
Browse files Browse the repository at this point in the history
  • Loading branch information
FR-vdash-bot committed Jan 12, 2023
1 parent 9b2f42b commit e43514a
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/Data/Nat/WithBot.lean
Original file line number Diff line number Diff line change
Expand Up @@ -56,10 +56,10 @@ theorem add_eq_three_iff {n m : WithBot ℕ} :
#align nat.with_bot.add_eq_three_iff Nat.WithBot.add_eq_three_iff

@[simp]
theorem coe_nonneg {n : ℕ} : 0 ≤ (n : WithBot ℕ) := by
theorem coe_nonneg' {n : ℕ} : 0 ≤ (n : WithBot ℕ) := by
rw [← WithBot.coe_zero]
exact WithBot.coe_le_coe.mpr (Nat.zero_le n)
#align nat.with_bot.coe_nonneg Nat.WithBot.coe_nonneg
#align nat.with_bot.coe_nonneg Nat.WithBot.coe_nonneg'

@[simp]
theorem lt_zero_iff (n : WithBot ℕ) : n < 0 ↔ n = ⊥ := by
Expand Down

0 comments on commit e43514a

Please sign in to comment.