Files
colloquium-lean/ColloquiumLean/ContinuousSquare.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
798 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
variable
{x : } {y : }
-- Definition: Function (f : ) is continuous at (x₀ : )
def continuous_at (f : ) (x₀ : ) :=
ε > 0, δ > 0, x, |x - x₀| < δ |f x - f x₀| < ε
-- Three lemmas from the lean mathematical library
example : 0 < x 0 < x := sqrt_pos.2
example : x ^ 2 < y (-y < x) (x < y) := sq_lt
example : |x| < y -y < x x < y := abs_lt
-- The square function
def squareFct : := fun x x ^ 2
theorem continuous_at_squareFct :
continuous_at squareFct 0 := by
unfold continuous_at
intro e he
use e
constructor
· apply sqrt_pos.2
exact he
· intro x hx
simp_all [squareFct]
apply sq_lt.2
apply abs_lt.1
exact hx