Demostraciones de "f⁻¹(u ∩ v) = f⁻¹(u) ∩ f⁻¹(v)"
Demostrar con Lean4 y con Isabelle/HOL que
f⁻¹(u ∩ v) = f⁻¹(u) ∩ f⁻¹(v)
Para ello, completar la siguiente teoría de Lean4:
import Mathlib.Data.Set.Function variable {α β : Type _} variable (f : α → β) variable (u v : Set β) open Set example : f ⁻¹' (u ∩ v) = f ⁻¹' u ∩ f ⁻¹' v := by sorry
y la siguiente teoría de Iasbelle/HOL:
theory Imagen_inversa_de_la_interseccion imports Main begin lemma "f -` (u ∩ v) = f -` u ∩ f -` v" sorry end