Skip to content

Commit

Permalink
chore(SuccPred/Limit): rename 2 lemmas
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Oct 30, 2024
1 parent 926fb9e commit e3b5f4d
Showing 1 changed file with 7 additions and 6 deletions.
13 changes: 7 additions & 6 deletions Mathlib/Order/SuccPred/Limit.lean
Original file line number Diff line number Diff line change
Expand Up @@ -53,10 +53,10 @@ theorem not_isSuccPrelimit_iff_exists_covBy (a : α) : ¬IsSuccPrelimit a ↔
alias not_isSuccLimit_iff_exists_covBy := not_isSuccPrelimit_iff_exists_covBy

@[simp]
theorem isSuccPrelimit_of_dense [DenselyOrdered α] (a : α) : IsSuccPrelimit a := fun _ => not_covBy
theorem IsSuccPrelimit.of_dense [DenselyOrdered α] (a : α) : IsSuccPrelimit a := fun _ => not_covBy

@[deprecated isSuccPrelimit_of_dense (since := "2024-09-05")]
alias isSuccLimit_of_dense := isSuccPrelimit_of_dense
@[deprecated (since := "2024-09-30")] alias isSuccPrelimit_of_dense := IsSuccPrelimit.of_dense
@[deprecated (since := "2024-09-05")] alias isSuccLimit_of_dense := IsSuccPrelimit.of_dense

end LT

Expand Down Expand Up @@ -327,10 +327,11 @@ theorem not_isPredPrelimit_iff_exists_covBy (a : α) : ¬IsPredPrelimit a ↔
@[deprecated not_isPredPrelimit_iff_exists_covBy (since := "2024-09-05")]
alias not_isPredLimit_iff_exists_covBy := not_isPredPrelimit_iff_exists_covBy

theorem isPredPrelimit_of_dense [DenselyOrdered α] (a : α) : IsPredPrelimit a := fun _ => not_covBy
@[simp]
theorem IsPredPrelimit.of_dense [DenselyOrdered α] (a : α) : IsPredPrelimit a := fun _ => not_covBy

@[deprecated isPredPrelimit_of_dense (since := "2024-09-05")]
alias isPredLimit_of_dense := isPredPrelimit_of_dense
@[deprecated (since := "2024-09-30")] alias isPredPrelimit_of_dense := IsPredPrelimit.of_dense
@[deprecated (since := "2024-09-05")] alias isPredLimit_of_dense := IsPredPrelimit.of_dense

@[simp]
theorem isSuccPrelimit_toDual_iff : IsSuccPrelimit (toDual a) ↔ IsPredPrelimit a := by
Expand Down

0 comments on commit e3b5f4d

Please sign in to comment.