(* Imagen_inversa_de_la_imagen.thy -- s ⊆ f⁻¹[f[s]] -- José A. Alonso Jiménez -- Sevilla, 7-junio-2021 -- ------------------------------------------------------------------ *) (* --------------------------------------------------------------------- -- Demostrar que si s es un subconjunto del dominio de la función f, -- entonces s está contenido en la imagen inversa de la imagen de s por -- f; es decir, -- s \ f⁻¹[f[s]] -- ------------------------------------------------------------------- *) theory Imagen_inversa_de_la_imagen imports Main begin (* 1\ demostración *) lemma "s \ f -` (f ` s)" proof (rule subsetI) fix x assume "x \ s" then have "f x \ f ` s" by (simp only: imageI) then show "x \ f -` (f ` s)" by (simp only: vimageI) qed (* 2\ demostración *) lemma "s \ f -` (f ` s)" proof fix x assume "x \ s" then have "f x \ f ` s" by simp then show "x \ f -` (f ` s)" by simp qed (* 3\ demostración *) lemma "s \ f -` (f ` s)" by auto end