Si f es suprayectiva, entonces u ⊆ f[f⁻¹[u]]
Demostrar con Lean4 y con Isabelle/HOL que si \(f\) es suprayectiva, entonces \[ u ⊆ f[f⁻¹[u]] \]
Para ello, completar la siguiente teoría de Lean4:
import Mathlib.Data.Set.Function open Set Function variable {α β : Type _} variable (f : α → β) variable (u : Set β) example (h : Surjective f) : u ⊆ f '' (f⁻¹' u) := by sorry
y la siguiente teoría de Isabelle/HOL:
theory Imagen_de_imagen_inversa_de_aplicaciones_suprayectivas imports Main begin lemma assumes "surj f" shows "u ⊆ f ` (f -` u)" sorry end