You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
{{ message }}
This repository has been archived by the owner on Oct 14, 2023. It is now read-only.
Reduced the issue to a self-contained, reproducible test case.
Description
ASCII angle brackets of the form (| ... |) and pretty angle brackets ⟨ ... ⟩ appear to take different precedence, and so behave differently.
Steps to Reproduce
Attempt to run lean against the following file (which is the example I have on hand and not necessarily a MWE)
variables (A : Type) (p q : A -> Prop)
variable a : A
example : (exists x , p x \/ q x) -> (exists x , p x ) \/ (exists x , q x) :=
assume (| a, (pqa : p a \/ q a) |),
or.elim pqa
(
assume hpa : p a, or.inl ⟨a, hpa⟩
)
(
assume hqa : q a, or.inr (|a, hqa|)
--assume hqa : q a, or.inr ( (|a, hqa|) )
--assume hqa : q a, or.inr ⟨a, hqa⟩
)
Expected behavior: No output
Actual behavior: Error output
/tmp/t.lean:12:33: error: invalid expression, `)` expected
/tmp/t.lean:12:33: error: command expected
/tmp/t.lean:7:4: error: type mismatch at application
or.elim pqa (λ (hpa : p a), or.inl (Exists.intro a hpa)) (λ (hqa : q a), or.inr)
term
λ (hqa : q a), or.inr
has type
Π (hqa : q a), ?m_1[hqa] → ?m_2[hqa] ∨ ?m_1[hqa]
but is expected to have type
q a → ((∃ (x : A), p x) ∨ ∃ (x : A), q x)
This goes away if either of the two commented out lines is substituted back in.
Prerequisites
or feature requests.
Description
ASCII angle brackets of the form
(| ... |)
and pretty angle brackets⟨ ... ⟩
appear to take different precedence, and so behave differently.Steps to Reproduce
lean
against the following file (which is the example I have on hand and not necessarily a MWE)Expected behavior: No output
Actual behavior: Error output
This goes away if either of the two commented out lines is substituted back in.
Reproduces how often: Always
Versions
Operating system
The text was updated successfully, but these errors were encountered: