Skip to content

Commit

Permalink
deprecations
Browse files Browse the repository at this point in the history
  • Loading branch information
vihdzp committed Oct 12, 2024
1 parent cc9d992 commit c17bf63
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions Mathlib/SetTheory/Surreal/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -244,6 +244,12 @@ theorem insertRight {x x' : PGame} (x_num : x.Numeric) (x'_num : x'.Numeric)

end Numeric

@[deprecated Numeric.insertLeft (since := "2024-10-11")]
alias insertLeft_numeric := Numeric.insertLeft

@[deprecated Numeric.insertRight (since := "2024-10-11")]
alias insertRight_numeric := Numeric.insertRight

/-- Pre-games defined by natural numbers are numeric. -/
theorem numeric_nat : ∀ n : ℕ, Numeric n
| 0 => numeric_zero
Expand Down

0 comments on commit c17bf63

Please sign in to comment.