Files
colloquium-lean/ColloquiumLean/ContinuousLimit.lean
Stefan Kebekus 50952410a4
Some checks failed
Create Release / Add Lean release tag (push) Has been cancelled
Lean Action CI / build (push) Has been cancelled
Working
2025-09-29 14:53:44 +02:00

25 lines
885 B
Lean4
Raw Blame History

This file contains ambiguous Unicode characters

This file contains Unicode characters that might be confused with other characters. If you think that this is intentional, you can safely ignore this warning. Use the Escape button to reveal them.

-- Library Import: Basic facts about real numbers
import Mathlib
open Real
-- Definition: Function (f : ) is continuous at (x₀ : )
def continuous_at (f : ) (x₀ : ) :=
ε > 0, δ > 0, x, |x - x₀| < δ |f x - f x₀| < ε
-- Definition: Sequence (u : ) converges to limit (l : )
def seq_limit (u : ) (l : ) :=
ε > 0, N, n N, |u n - l| < ε
-- In the following, f is a function, u is a sequence, and x₀ a real number
variable
{f : } {u : } {x₀ : }
/-
Theorem "Continuity and Limits": If the function f is continuous at x₀ and u
is a sequence converging to x₀, then the sequence f ∘ u converges to f (x₀).
-/
theorem continuity_and_limits (hyp_f : continuous_at f x₀) (hyp_u : seq_limit u x₀) :
seq_limit (f u) (f x₀) := by
sorry