Skip to content
This repository has been archived by the owner on Oct 10, 2023. It is now read-only.

Commit

Permalink
Add lim_le hint (#51)
Browse files Browse the repository at this point in the history
lemma lim_le is in answer and tuto_lib but not in exercise hint
  • Loading branch information
fzyzcjy committed Dec 26, 2022
1 parent c17f27f commit 79a6872
Show file tree
Hide file tree
Showing 2 changed files with 8 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/exercises/09_limits_final.lean
Original file line number Diff line number Diff line change
Expand Up @@ -71,6 +71,10 @@ and their easy consequences:
limit_const_sub_inv_succ (x : ℝ) : seq_limit (λ n, x - 1/(n+1)) x
as well as:
lim_le (hu : seq_limit u x) (ineg : ∀ n, u n ≤ y) : x ≤ y
The structure of the proof is offered. It features a new tactic:
`choose` which invokes the axiom of choice (observing the tactic state before and
after using it should be enough to understand everything).
Expand Down
4 changes: 4 additions & 0 deletions src/solutions/09_limits_final.lean
Original file line number Diff line number Diff line change
Expand Up @@ -81,6 +81,10 @@ and their easy consequences:
limit_const_sub_inv_succ (x : ℝ) : seq_limit (λ n, x - 1/(n+1)) x
as well as:
lim_le (hu : seq_limit u x) (ineg : ∀ n, u n ≤ y) : x ≤ y
The structure of the proof is offered. It features a new tactic:
`choose` which invokes the axiom of choice (observing the tactic state before and
after using it should be enough to understand everything).
Expand Down

0 comments on commit 79a6872

Please sign in to comment.