Demostraciones de "f[s ∩ t] ⊆ f[s] ∩ f[t]"
Demostrar con Lean4 y con Isabelle/HOL que \[ f[s ∩ t] ⊆ f[s] ∩ f[t] \]
Para ello, completar la siguiente teoría de Lean4:
import Mathlib.Data.Set.Function import Mathlib.Tactic open Set variable {α β : Type _} variable (f : α → β) variable (s t : Set α) example : f '' (s ∩ t) ⊆ f '' s ∩ f '' t := by sorry
y la siguiente teoría de Isabelle/HOL:
theory Imagen_de_la_interseccion imports Main begin lemma "f ` (s ∩ t) ⊆ f ` s ∩ f ` t" sorry end