Zulip Chat Archive

Stream: maths

Topic: filter.mem_map


Nicolò Cavalleri (Jun 10 2021 at 15:57):

Is there any reason that mem_map is in mathlib in this form

@[simp] lemma mem_map : t  map m f  {x | m x  t}  f := iff.rfl

and not in this form

@[simp] lemma mem_map : t  map m f  m ⁻¹' t  f := iff.rfl

?

Yakov Pechersky (Jun 10 2021 at 16:02):

Does set.preimage work here?

Patrick Massot (Jun 10 2021 at 16:02):

This is not the type of t

Patrick Massot (Jun 10 2021 at 16:02):

I don't see any reason why this lemma should be stated like that.

Patrick Massot (Jun 10 2021 at 16:02):

You should try to change it and see whether it breaks anything

Yakov Pechersky (Jun 10 2021 at 16:05):

Ah yes, t : \beta. And I bet it would not work because t is not a set _

Yakov Pechersky (Jun 10 2021 at 16:05):

You could try m ⁻¹' {t}?

Patrick Massot (Jun 10 2021 at 16:06):

Why do you say t is not a set?

Yakov Pechersky (Jun 10 2021 at 16:06):

But I bet the simp-normal form is the one as it is stated

Yakov Pechersky (Jun 10 2021 at 16:06):

Patrick, you are again correct, and I am confused.

Nicolò Cavalleri (Jun 10 2021 at 16:08):

Patrick Massot said:

I don't see any reason why this lemma should be stated like that.

Like what sorry? You don't see why it is how it is or why it should be how I want it?

Patrick Massot (Jun 10 2021 at 16:09):

I don't why it is stated the way it's currently stated. Maybe this isn't clearer. I mean I agree with you.

Nicolò Cavalleri (Jun 10 2021 at 16:09):

Ok thanks I will PR then


Last updated: Dec 20 2023 at 11:08 UTC