Files
colloquium-lean/ColloquiumLean/ContinuousLimitSolution.lean
Stefan Kebekus ea169e4c3e
Some checks failed
Lean Action CI / build (push) Has been cancelled
Initial checkout
2025-09-15 14:41:27 +02:00

36 lines
1.0 KiB
Lean4
Raw Permalink 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.Data.Real.Basic
open Real
-- Definition: Function (f : ) is continuous at (x₀ : )
def continuous (f : ) (x₀ : ) :=
ε > 0, δ > 0, x, |x - x₀| < δ |f x - f x₀| < ε
-- Definition: Sequence (u : ) converges to limit (l : )
def 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: If f is continuous at x₀ and the sequence u converges to x₀, then
-- the sequence f ∘ u converges to f x₀.
theorem continuity_and_limits
(hyp_f : continuous f x₀) (hyp_u : limit u x₀) :
limit (f u) (f x₀) := by
unfold limit at *
unfold continuous at *
intro ε
obtain δ, h₁δ, h₂δ := hyp_f ε
obtain N, hN := hyp_u δ h₁δ
use N
intro n hn
apply h₂δ
apply hN
exact hn