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
In the example below, Prod.continuous is a partially-typed declaration name.
structure ContinuousSMul (M X : Type) : Prop where
structure ContinuousAdd (X : Type) : Prop where
theorem Prod.continuousSMul {M X Y : Type} : ContinuousSMul M (X × Y) := ⟨⟩
theorem Prod.continuousAdd {X Y : Type} : ContinuousAdd (X × Y) := ⟨⟩
example : (ContinuousSMul Nat (Nat × Nat)) ∧ (ContinuousAdd (Nat × Nat)) := by
exact ⟨Prod.continuousSMul, Prod.continuous⟩ -- put cursor after `s` in `Prod.continuous`
-- and ctrl-space fails for me
I would expect autocompletion in VS Code to offer me e.g. Prod.continuousAdd (the thing which will close the goal), but for me it offers nothing:
Fixes#4455, fixes#4705, fixes#5219
Also fixes a minor bug where a dot in brackets would report incorrect
completions instead of no completions.
---------
Co-authored-by: Sebastian Ullrich <sebasti@nullri.ch>
Fixesleanprover#4455, fixesleanprover#4705, fixesleanprover#5219
Also fixes a minor bug where a dot in brackets would report incorrect
completions instead of no completions.
---------
Co-authored-by: Sebastian Ullrich <sebasti@nullri.ch>
Prerequisites
Please put an X between the brackets as you perform the following steps:
https://github.com/leanprover/lean4/issues
Avoid dependencies to Mathlib or Batteries.
https://live.lean-lang.org/#project=lean-nightly
(You can also use the settings there to switch to “Lean nightly”)
Description
In the example below,
Prod.continuous
is a partially-typed declaration name.I would expect autocompletion in VS Code to offer me e.g.
Prod.continuousAdd
(the thing which will close the goal), but for me it offers nothing:Context
https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/autocompletion.20problem/near/466255717
Steps to Reproduce
s
inProd.continuous
Expected behavior: [Clear and concise description of what you expect to happen]
Suggestions pop up e.g.
Prod.continuousSMul
,Prod.continuousAdd
.Actual behavior: [Clear and concise description of what actually happens]
No suggestions.
Versions
Lean (version 4.11.0-rc1, x86_64-unknown-linux-gnu, commit daa2218, Release)
Impact
Add 👍 to issues you consider important. If others are impacted by this issue, please ask them to add 👍 to it.
The text was updated successfully, but these errors were encountered: