Zulip Chat Archive
Stream: Is there code for X?
Topic: inner product space eq
Moritz Doll (Jul 13 2022 at 20:59):
Is this lemma in mathlib? I haven't found it, but I feel like it should exist
import analysis.inner_product_space.basic
variables (π : Type*) {E : Type*}
variables [is_R_or_C π] [inner_product_space π E]
example {x x' : E} (h : β y : E, inner x y = (inner x' y : π)) : x = x' :=
begin
specialize h (x - x'),
rw [βsub_eq_zero, βinner_self_eq_zero, inner_sub_left, sub_eq_zero],
exact h,
end
Eric Wieser (Jul 13 2022 at 21:39):
Maybe it's named something like docs#inner_left_inj?
FrΓ©dΓ©ric Dupuis (Jul 13 2022 at 21:48):
docs#inner_product_space.ext_inner_right
Eric Wieser (Jul 13 2022 at 22:03):
I guess we don't have the version that says function.injective (inner x)
?
Wrenna Robson (Jul 14 2022 at 06:27):
Isn't that docs#inner_product_space.ext_inner_left?
Wrenna Robson (Jul 14 2022 at 06:27):
I guess maybe that puts the quantifier in a different place.
Last updated: Dec 20 2023 at 11:08 UTC