Zulip Chat Archive
Stream: new members
Topic: Unexpected `#guard_msgs` error
Asei Inoue (Jan 08 2024 at 05:54):
Why the following code raise an error ":cross_mark: Docstring on #guard_msgs
does not match generated message:"?
import Mathlib.Tactic.Common
/-- info: inductive Or : Prop → Prop → Prop
number of parameters: 2
constructors:
Or.inl : ∀ {a b : Prop}, a → a ∨ b
Or.inr : ∀ {a b : Prop}, b → a ∨ b -/
#guard_msgs in
#print Or
Asei Inoue (Jan 08 2024 at 06:50):
I think #guard_msgs
should ignore whitespace and breakline:
import Mathlib.Tactic
variable (α : Type)
/-! the following is correct -/
/--
error: failed to synthesize instance Inv α
-/
#guard_msgs in
#check (_ : α)⁻¹
/-! the following is **not** correct -/
/--
error: failed to synthesize instance Inv α
-/
#guard_msgs in
#check (_ : α)⁻¹
Asei Inoue (Jan 08 2024 at 07:02):
I think there are other people besides me who have problems with this behaviour of #guard_msgs
.
Last updated: May 02 2025 at 03:31 UTC