Zulip Chat Archive
Stream: new members
Topic: convert to term mode
Ashwin Iyengar (Feb 12 2021 at 13:54):
Hi, I don't really understand term mode. Right now this works:
noncomputable def add (f g : mv_restricted_power_series σ R) : mv_restricted_power_series σ R := ⟨f.1 + g.1, begin
have x := tendsto.add f.2 g.2,
simp at x,
exact x,
end⟩
But this doesn't work:
noncomputable def add (f g : mv_restricted_power_series σ R) : mv_restricted_power_series σ R := ⟨f.1 + g.1, tendsto.add f.2 g.2⟩
So how do I convert the first block into term mode and incorporate the simp?
Yakov Pechersky (Feb 12 2021 at 13:59):
Does this work for you?
noncomputable def add (f g : mv_restricted_power_series σ R) : mv_restricted_power_series σ R := ⟨f.1 + g.1, by simpa using tendsto.add f.2 g.2⟩
Ashwin Iyengar (Feb 12 2021 at 14:01):
Yes, thanks! And I just found the documentation for by
, so that's helpful.
Last updated: Dec 20 2023 at 11:08 UTC