Files
colloquium-lean/ColloquiumLean/ContinuousLimit.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

23 lines
669 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.

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₀ : }
lemma continuity_and_limits
(hyp_f : continuous_at f x₀) (hyp_u : seq_limit u x₀) :
seq_limit (f u) (f x₀) := by
sorry