Zulip Chat Archive
Stream: mathlib4
Topic: apply (config := { instances := false })
Kevin Buzzard (May 13 2023 at 17:30):
mathlib3port is turning apply_with foo { instances := ff },
into apply (config := { instances := false }) foo
, which is barfing with a syntax error (expected ')', ',' or ':'
). Is apply
config
urable? I'm assuming not and will work around accordingly.
Kyle Miller (May 13 2023 at 17:35):
It looks like you have to import Mathlib.Tactic.ApplyWith
Adam Topaz (May 13 2023 at 17:43):
But note that docs4#Lean.Meta.ApplyConfig doesn't have an instances
field.
Last updated: Dec 20 2023 at 11:08 UTC