Skip to content

Commit

Permalink
docs(order/order_iso_nat): Added note on `exists_increasing_or_noninc…
Browse files Browse the repository at this point in the history
…reasing_subseq` (#12239)
  • Loading branch information
vihdzp committed Feb 23, 2022
1 parent 162d060 commit 3e2df83
Showing 1 changed file with 2 additions and 0 deletions.
2 changes: 2 additions & 0 deletions src/order/order_iso_nat.lean
Expand Up @@ -140,6 +140,8 @@ begin
or.intro_left _ (λ n, (nat.find_spec (h (g' n))).2)⟩ }
end

/-- This is the infinitary Erdős–Szekeres theorem, and an important lemma in the usual proof of
Bolzano-Weierstrass for `ℝ`. -/
theorem exists_increasing_or_nonincreasing_subseq
{α : Type*} (r : α → α → Prop) [is_trans α r] (f : ℕ → α) :
∃ (g : ℕ ↪o ℕ), (∀ m n : ℕ, m < n → r (f (g m)) (f (g n))) ∨
Expand Down

0 comments on commit 3e2df83

Please sign in to comment.