Skip to content

Commit

Permalink
feat: make Set.mem_image_equiv a simp lemma (#5644)
Browse files Browse the repository at this point in the history
Not certain about this one.

It's useful for me (experimenting with `UnivLE`), and arguably this is a better simp normal form since `''` is relatively hard to reason about, but I'm not certain how it interacts with everything else. Let's see what CI says.



Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed Jul 1, 2023
1 parent a9b3aae commit b856949
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Subobject/Lattice.lean
Expand Up @@ -707,7 +707,7 @@ theorem sSup_le {A : C} (s : Set (Subobject A)) (f : Subobject A) (k : ∀ g ∈
· refine' Sigma.desc _
rintro ⟨g, m⟩
refine' underlying.map (homOfLE (k _ _))
simpa [symm_apply_mem_iff_mem_image] using m
simpa using m
· ext
dsimp [smallCoproductDesc]
simp
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Logic/Equiv/Set.lean
Expand Up @@ -44,6 +44,7 @@ protected theorem image_eq_preimage {α β} (e : α ≃ β) (s : Set α) : e ''
Set.ext fun _ => mem_image_iff_of_inverse e.left_inv e.right_inv
#align equiv.image_eq_preimage Equiv.image_eq_preimage

@[simp 1001]
theorem _root_.Set.mem_image_equiv {α β} {S : Set α} {f : α ≃ β} {x : β} :
x ∈ f '' S ↔ f.symm x ∈ S :=
Set.ext_iff.mp (f.image_eq_preimage S) x
Expand Down

0 comments on commit b856949

Please sign in to comment.