Skip to content

Commit 7a11b9f

Browse files
committed
feat(PNat/Basic): add three lemmas (#12479)
Three small lemmata in support of further PNat proofs
1 parent cf57f9b commit 7a11b9f

File tree

1 file changed

+7
-0
lines changed

1 file changed

+7
-0
lines changed

Mathlib/Data/PNat/Basic.lean

Lines changed: 7 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -314,6 +314,13 @@ theorem pow_coe (m : ℕ+) (n : ℕ) : ↑(m ^ n) = (m : ℕ) ^ n :=
314314
rfl
315315
#align pnat.pow_coe PNat.pow_coe
316316

317+
/-- b is greater one if any a is less than b -/
318+
theorem one_lt_of_lt {a b : ℕ+} (hab : a < b) : 1 < b := bot_le.trans_lt hab
319+
320+
theorem add_one (a : ℕ+) : a + 1 = succPNat a := rfl
321+
322+
theorem lt_succ_self (a : ℕ+) : a < succPNat a := lt.base a
323+
317324
/-- Subtraction a - b is defined in the obvious way when
318325
a > b, and by a - b = 1 if a ≤ b.
319326
-/

0 commit comments

Comments
 (0)