Zulip Chat Archive
Stream: general
Topic: (u : Fin 2) → (Even u ↔ Even u.val)
Iván Renison (Dec 10 2023 at 21:00):
Hello, I'm trying to prove this:
theorem aux28 (u : Fin 2) : Even u ↔ Even u.val := sorry
Witch I think should also be valid for Fin n
, but I'm not being able to prove it.
I was able to reduce it to having to prove this:
theorem aux33 : ¬Even (1 : Fin 2) := sorry
But i'm not able to prove that neither
How could I do?
Ruben Van de Velde (Dec 10 2023 at 21:14):
Not for odd :
example : ¬∀ (u : Fin 5), Even u ↔ Even u.val := by
simp
use 3
simp
use 4
simp
Thomas Murrills (Dec 10 2023 at 21:17):
theorem aux33 : ¬Even (1 : Fin 2) := by unfold Even; decide
works. (I feel like decide
should work without the unfold
; presumably we just could do with another instance somewhere?)
Iván Renison (Dec 10 2023 at 21:19):
Thank you
Yury G. Kudryashov (Dec 10 2023 at 21:45):
I'm working on
lemma Fin.even_iff {n : ℕ} {k : Fin n} : Even k ↔ Odd n ∨ Even k.val := by
Last updated: Dec 20 2023 at 11:08 UTC