Zulip Chat Archive
Stream: new members
Topic: exacts
Nicolò Cavalleri (Jun 26 2021 at 17:32):
Why does not this work?
import data.equiv.local_equiv
open set
variables {α : Type*} {β : Type*} {γ : Type*} {δ : Type*}
variables (e : local_equiv α β) (e' : local_equiv β γ)
variables {e} {s : set α} {t : set β} {x : α} {y : β}
lemma source_inter_preimage_target_inter (s : set β) :
  e.source ∩ (e ⁻¹' (e.target ∩ s)) = e.source ∩ (e ⁻¹' s) :=
begin
  refine ext_iff.mpr (λ x, ⟨λ hx, _, λ hx, _⟩),
  simp only [mem_inter_eq, mem_preimage] at *;
  exacts [⟨hx.1, hx.2.2⟩, ⟨hx.1, e.map_source hx.1, hx.2⟩], --exacts?
end
Adam Topaz (Jun 26 2021 at 17:38):
Is this missing an import?
Adam Topaz (Jun 26 2021 at 17:38):
The code doesn't work for me
Nicolò Cavalleri (Jun 26 2021 at 18:04):
Sorry, I pasted the wrong import, now it should work
Kyle Miller (Jun 26 2021 at 18:04):
It's weird, splitting it into two exact tactics works
Kyle Miller (Jun 26 2021 at 18:05):
I'm also not sure why the exact tactics work
Nicolò Cavalleri (Jun 26 2021 at 18:05):
Yes that's my point I mean it probably has something to do with the fact that I use an implicit construtctor?
Adam Topaz (Jun 26 2021 at 18:05):
You have a semicolon. Change it to a comma
Kyle Miller (Jun 26 2021 at 18:06):
Oh, I completely missed the ;.  Exacts should work when there are multiple goals.
Kyle Miller (Jun 26 2021 at 18:06):
When it's a ;, it means it applies the tactic to each goal that the previous tactic has created.
Nicolò Cavalleri (Jun 26 2021 at 18:12):
Oh right!! I meant to put it on the previous line! I wanted to apply the simp to both goals!
Nicolò Cavalleri (Jun 26 2021 at 18:12):
Thanks to both!
Nicolò Cavalleri (Jun 26 2021 at 18:14):
And thanks to this I realized the simp is not needed.
Kyle Miller (Jun 26 2021 at 19:55):
@Nicolò Cavalleri You probably already worked this out after removing the simp, but you can condense it down to a one-liner term-mode proof:
lemma source_inter_preimage_target_inter (s : set β) :
  e.source ∩ (e ⁻¹' (e.target ∩ s)) = e.source ∩ (e ⁻¹' s) :=
ext (λ x, ⟨λ hx, ⟨hx.1, hx.2.2⟩, λ hx, ⟨hx.1, e.map_source hx.1, hx.2⟩⟩)
(note that set.ext_iff.mpr is set.ext)
Nicolò Cavalleri (Jun 26 2021 at 19:56):
Yes I know! I already pushed it to mathlib! Thanks anyways!
Nicolò Cavalleri (Jun 26 2021 at 19:56):
Kyle Miller said:
(note that
set.ext_iff.mprisset.ext)
I did not know this though! Thanks!
Last updated: May 02 2025 at 03:31 UTC