We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
f '' s = f ⁻¹' s
f
1 parent f5dca22 commit bfadd55Copy full SHA for bfadd55
Mathlib/Data/Set/Image.lean
@@ -351,6 +351,10 @@ theorem image_eq_preimage_of_inverse {f : α → β} {g : β → α} (h₁ : Lef
351
funext fun s =>
352
Subset.antisymm (image_subset_preimage_of_inverse h₁ s) (preimage_subset_image_of_inverse h₂ s)
353
354
+theorem _root_.Function.Involutive.image_eq_preimage {f : α → α} (hf : f.Involutive) :
355
+ image f = preimage f :=
356
+ image_eq_preimage_of_inverse hf.leftInverse hf.rightInverse
357
+
358
theorem mem_image_iff_of_inverse {f : α → β} {g : β → α} {b : β} {s : Set α} (h₁ : LeftInverse g f)
359
(h₂ : RightInverse g f) : b ∈ f '' s ↔ g b ∈ s := by
360
rw [image_eq_preimage_of_inverse h₁ h₂]; rfl
0 commit comments