Zulip Chat Archive
Stream: mathlib4
Topic: Cases does not change assumptions
David Ang (Jun 21 2023 at 20:00):
I noticed that sometimes cases
does not modify assumptions - is this intentional?
import Mathlib.Data.Polynomial.Degree.Definitions
example (R : Type) [CommRing R] (f : Polynomial R) (h : f.degree = some 0) : f.degree = some 0 := by
cases f.degree with
| none => rfl -- fails, because `h` did not get changed
| some n => rfl -- fails, because `h` did not get changed
I could certainly do revert h
and intro h
afterwards, or cases h : f.degree
and rw [h]
at necessary places, but both seem redundant.
Grant Barkley (Jun 21 2023 at 22:27):
Last updated: Dec 20 2023 at 11:08 UTC