Skip to content

Commit

Permalink
chore: classify new instance porting notes (#11433)
Browse files Browse the repository at this point in the history
Classifies by adding issue number #10754 to porting notes claiming "new instance".
  • Loading branch information
pitmonticone authored and atarnoam committed Apr 16, 2024
1 parent 8655f13 commit f22bad9
Show file tree
Hide file tree
Showing 4 changed files with 4 additions and 4 deletions.
2 changes: 1 addition & 1 deletion Mathlib/Data/Nat/PartENat.lean
Original file line number Diff line number Diff line change
Expand Up @@ -680,7 +680,7 @@ def ofENat : ℕ∞ → PartENat :=
| Option.none => none
| Option.some n => some n

-- Porting note: new
-- Porting note (#10754): new instance
instance : Coe ℕ∞ PartENat := ⟨ofENat⟩

-- Porting note: new. This could probably be moved to tests or removed.
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/PNat/Defs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -44,7 +44,7 @@ instance coePNatNat : Coe ℕ+ ℕ :=
instance : Repr ℕ+ :=
fun n n' => reprPrec n.1 n'⟩

-- Porting note: New instance not in Lean3
--Porting note (#10754): New instance not in Lean3
instance (n : ℕ) : OfNat ℕ+ (n+1) :=
⟨⟨n + 1, Nat.succ_pos n⟩⟩

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/InformationTheory/Hamming.lean
Original file line number Diff line number Diff line change
Expand Up @@ -450,7 +450,7 @@ theorem nndist_eq_hammingDist (x y : Hamming β) :
rfl
#align hamming.nndist_eq_hamming_dist Hamming.nndist_eq_hammingDist

-- Porting note: new
-- Porting note (#10754): new instance
instance : DiscreteTopology (Hamming β) := ⟨rfl⟩

instance : MetricSpace (Hamming β) := .ofT0PseudoMetricSpace _
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Init/Order/Defs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -129,7 +129,7 @@ theorem gt_of_ge_of_gt {a b c : α} (h₁ : a ≥ b) (h₂ : b > c) : a > c :=
lt_of_lt_of_le h₂ h₁
#align gt_of_ge_of_gt gt_of_ge_of_gt

-- Porting note: new
-- Porting note (#10754): new instance
instance (priority := 900) : @Trans α α α LE.le LE.le LE.le := ⟨le_trans⟩
instance (priority := 900) : @Trans α α α LT.lt LT.lt LT.lt := ⟨lt_trans⟩
instance (priority := 900) : @Trans α α α LT.lt LE.le LT.lt := ⟨lt_of_lt_of_le⟩
Expand Down

0 comments on commit f22bad9

Please sign in to comment.