Zulip Chat Archive
Stream: new members
Topic: ifinish
Michael Beeson (Sep 12 2020 at 06:56):
ifinish doesn't succeed with this simple proposition:
example: ∀ (A B:Prop), (A → B) → ((A ∧ B) ↔ A)
This is not a question, or even a complaint really, I'm just trying to get familiar enough with ifinish so as to know
whether to expect it to succeed or not. I thought it would do this one.
Kenny Lau (Sep 12 2020 at 07:06):
it does for me
Michael Beeson (Sep 12 2020 at 07:31):
lemma lemma11helper1: ∀ (A B:Prop), (A → B) → ((A ∧ B) ↔ A) :=
assume A B,
begin
ifinish,
end
produces
solve1 tactic failed, focused goal has not been solved
state:
A B : Prop,
a : A → B,
f : Prop,
a_1 : (A ∧ B ↔ A) → f
⊢ f
So please post your corresponding input and successful output.
Markus Himmel (Sep 12 2020 at 07:32):
It works with current Lean and mathlib:
Michael Beeson (Sep 12 2020 at 07:35):
Oh. So I should update lean using leanproject, I guess. I'm worried that some of my nice proofs might break then.
Last updated: Dec 20 2023 at 11:08 UTC