Monotonía de la imagen de conjuntos
Demostrar con Lean4 y con Isabelle/HOL que si \(s ⊆ t\), entonces \(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 (h : s ⊆ t) : f '' s ⊆ f '' t := by sorry
y la siguiente teoría de Isabelle/HOL:
theory Monotonia_de_la_imagen_de_conjuntos imports Main begin lemma assumes "s ⊆ t" shows "f ` s ⊆ f ` t" sorry end