We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent cf57f9b commit 7a11b9fCopy full SHA for 7a11b9f
Mathlib/Data/PNat/Basic.lean
@@ -314,6 +314,13 @@ theorem pow_coe (m : ℕ+) (n : ℕ) : ↑(m ^ n) = (m : ℕ) ^ n :=
314
rfl
315
#align pnat.pow_coe PNat.pow_coe
316
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
324
/-- Subtraction a - b is defined in the obvious way when
325
a > b, and by a - b = 1 if a ≤ b.
326
-/
0 commit comments