Zulip Chat Archive
Stream: Is there code for X?
Topic: findim_eq_one_iff
Scott Morrison (Apr 24 2021 at 10:36):
Do we have
lemma findim_eq_one_iff (v : V) (n : v ≠ 0) (h : ∀ w : V, ∃ c : K, w = c • v) :
findim K V = 1 :=
sorry
and/or an easy path to it?
Scott Morrison (Apr 24 2021 at 10:37):
Perhaps best to have
lemma findim_le_one_iff (v : V) (h : ∀ w : V, ∃ c : K, w = c • v) :
findim K V <= 1 :=
sorry
first?
Scott Morrison (Apr 24 2021 at 11:50):
Eric Wieser (Apr 24 2021 at 12:48):
Should we have these for dim
too?
Sebastien Gouezel (Apr 24 2021 at 12:50):
By the way, #7322 renames dim
and findim
to rank
and finrank
. If you don't like it, it is still time to voice your concerns on the PR page :-)
Last updated: Dec 20 2023 at 11:08 UTC