Zulip Chat Archive

Stream: new members

Topic: Error: don't know how to synthesize placeholder


Vasily Ilin (Sep 11 2021 at 23:01):

What is wrong here? I get "don't know how to synthesize placeholder" error.

example (a b c : ) (hc : c  0) (hab :  a  b) : b*c  a*c :=
begin
  rw  sub_nonneg,
  calc 0  (a-b)*c : mul_nonneg_of_nonpos_of_nonpos (by rwa sub_nonpos hab) hc,
     ... = a*c - b*c : by ring,
end

Kevin Buzzard (Sep 11 2021 at 23:01):

Can you post a #mwe? (All imports etc). It makes life easier for everyone else and it's the norm here.

Vasily Ilin (Sep 11 2021 at 23:04):

This is this file: https://github.com/leanprover-community/tutorials/blob/master/src/exercises/02_iff_if_and.lean. The only import is import data.real.basic as far as I can tell. So I guess the MWE is

import data.real.basic

example (a b c : ) (hc : c  0) (hab :  a  b) : b*c  a*c :=
begin
  rw  sub_nonneg,
  calc 0  (a-b)*c : mul_nonneg_of_nonpos_of_nonpos (by rwa sub_nonpos hab) hc,
     ... = a*c - b*c : by ring,
end

Vasily Ilin (Sep 11 2021 at 23:06):

Ah, it looks like it's the comma in calc... My bad!

Vasily Ilin (Sep 11 2021 at 23:07):

After deleting the comma and hab in rwas sub_nonpos hab everything works.

Kevin Buzzard (Sep 11 2021 at 23:09):

Yeah, sometimes the errors in calc mode can be pretty incomprehensible!


Last updated: Dec 20 2023 at 11:08 UTC