Tactics for topology #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Currently we have one domain-specific tactic for topology: continuity
.
continuity
tactic #
Automatically solve goals of the form continuous f
.
Mark lemmas with @[continuity]
to add them to the set of lemmas
used by continuity
.
continuity
solves goals of the form continuous f
by applying lemmas tagged with the
continuity
user attribute.
example {X Y : Type*} [topological_space X] [topological_space Y]
(f₁ f₂ : X → Y) (hf₁ : continuous f₁) (hf₂ : continuous f₂)
(g : Y → ℝ) (hg : continuous g) : continuous (λ x, (max (g (f₁ x)) (g (f₂ x))) + 1) :=
by continuity
will discharge the goal, generating a proof term like
((continuous.comp hg hf₁).max (continuous.comp hg hf₂)).add continuous_const
You can also use continuity!
, which applies lemmas with { md := semireducible }
.
The default behaviour is more conservative, and only unfolds reducible
definitions
when attempting to match lemmas with the goal.
continuity?
reports back the proof term it found.