Zulip Chat Archive

Stream: new members

Topic: Rewrite in lambda expr


Björn Fischer (May 22 2019 at 12:08):

Can I rewrite subterms of lambda expression (which depend on the argument)? rw does not find the pattern. Illustrative example:

variables (α : Type) (f : (α  α)  Prop)
lemma l (a : α) : id a = a := by refl

example : f (λ a, id a) := begin
    rw l, -- can't find pattern id ?m_2
end

Mario Carneiro (May 22 2019 at 12:11):

use dsimp or simp

Mario Carneiro (May 22 2019 at 12:11):

or conv


Last updated: Dec 20 2023 at 11:08 UTC