From: Holden Lee <hl422@cam.ac.uk>
Often, I have something I want to prove, say
f x = h x
and there is a simplification I want to use, say
P x => f x = g x
I would like Isabelle to replace the goal
by
Is there a simple way to do this (without a structured proof)? (Also note
that the x might be inside a !! quantifier, in which case I would want
would be replaced by
Thanks,
Holden
From: Lars Noschinski <noschinl@in.tum.de>
apply (subst <rule>)
-- Lars
From: René Thiemann <rene.thiemann@uibk.ac.at>
Dear Holden,
you might use trans[OF ...] as follows.
context
fixes P :: "'a => bool" and f g h :: "'a => 'a"
begin
lemma simp_me: "P x ==> f x = g x" sorry
lemma to_prove: "f x = h x"
apply (rule trans[OF simp_me])
sorry
end
Cheers,
René
From: Holden Lee <hl422@cam.ac.uk>
Thanks. One more wrinkle: In general I would like this to work if there
were other terms present. For example, to replace
with
Would this be possible?
Last updated: Nov 21 2024 at 12:39 UTC