File tree Expand file tree Collapse file tree 2 files changed +29
-0
lines changed
Expand file tree Collapse file tree 2 files changed +29
-0
lines changed Original file line number Diff line number Diff line change @@ -3656,6 +3656,7 @@ import Mathlib.Data.PNat.Factors
36563656import Mathlib.Data.PNat.Find
36573657import Mathlib.Data.PNat.Interval
36583658import Mathlib.Data.PNat.Notation
3659+ import Mathlib.Data.PNat.Order
36593660import Mathlib.Data.PNat.Prime
36603661import Mathlib.Data.PNat.Xgcd
36613662import Mathlib.Data.PSigma.Order
Original file line number Diff line number Diff line change 1+ /-
2+ Copyright (c) 2025 Javier Burroni. All rights reserved.
3+ Released under Apache 2.0 license as described in the file LICENSE.
4+ Authors: Javier Burroni
5+ -/
6+ import Mathlib.Algebra.Order.SuccPred
7+ import Mathlib.Data.PNat.Basic
8+
9+ /-!
10+ # Order related instances for `ℕ+`
11+ -/
12+
13+ namespace PNat
14+ open Nat
15+
16+ instance instSuccOrder : SuccOrder ℕ+ :=
17+ .ofSuccLeIff (· + 1 ) Iff.rfl
18+
19+ instance instSuccAddOrder : SuccAddOrder ℕ+ where
20+ succ_eq_add_one _ := rfl
21+
22+ instance instNoMaxOrder : NoMaxOrder ℕ+ where
23+ exists_gt n := ⟨n + 1 , lt_succ_self n⟩
24+
25+ @[simp]
26+ lemma succ_eq_add_one (n : ℕ+) : Order.succ n = n + 1 := rfl
27+
28+ end PNat
You can’t perform that action at this time.
0 commit comments