simplified README: this is for development version;
authorwenzelm
Sat, 02 Sep 2017 17:04:24 +0200
changeset 66596 c5bd8267d832
parent 66595 fa10b0f589c3
child 66597 53dcc7454221
simplified README: this is for development version;
src/Tools/VSCode/README.md
--- a/src/Tools/VSCode/README.md	Sat Sep 02 12:55:44 2017 +0200
+++ b/src/Tools/VSCode/README.md	Sat Sep 02 17:04:24 2017 +0200
@@ -1,23 +1,12 @@
 # Isabelle/PIDE for Visual Studio Code editor #
 
-* Extension for the editor ([TypeScript](extension/src/extension.ts))
-* Language Server protocol implementation ([Isabelle/Scala](src/server.scala))
-
-
-## Run ##
-
-* Extensions: search for "Isabelle", click "Install"
-
-* Preferences / User settings / edit settings.json: e.g.
-    `"isabelle.home": "/home/makarius/isabelle/repos"`
-
-* File / Open Folder: e.g. `src/HOL/Isar_Examples/` then open .thy files
-
-
 ## Debug ##
 
 * shell> `code src/Tools/VSCode/extension`
 
+* Preferences / User settings / edit settings.json: e.g.
+    `"isabelle.home": "/home/makarius/isabelle/repos"`
+
 * View / Debug / Launch Extension
 
 * File / Open Folder: e.g. `src/HOL/Isar_Examples/` then open .thy files
@@ -28,36 +17,3 @@
 * shell> `isabelle build_vscode`
 
 * Extensions / ... / Install from VSIX: `src/Tools/VSCode/extension/isabelle-X.Y.Z.vsix`
-
-
-## Relevant links ##
-
-### VSCode editor ###
-
-* https://code.visualstudio.com
-* https://code.visualstudio.com/docs/extensionAPI/extension-points
-* https://code.visualstudio.com/docs/extensions/example-language-server
-* https://github.com/Microsoft/vscode-languageserver-node-example
-* https://github.com/Microsoft/vscode
-
-
-### Protocol ###
-
-* https://code.visualstudio.com/blogs/2016/06/27/common-language-protocol
-* https://github.com/Microsoft/vscode-languageserver-node
-* https://github.com/Microsoft/language-server-protocol
-* https://github.com/Microsoft/language-server-protocol/blob/master/protocol.md
-* http://www.jsonrpc.org/specification
-* http://www.json.org
-
-
-### Similar projects ###
-
-* Lean Prover: https://github.com/leanprover/vscode-lean
-* Coq: https://github.com/siegebell/vscoq
-* OCaml: https://github.com/freebroccolo/vscode-reasonml
-* Scala: https://github.com/dragos/dragos-vscode-scala
-* Rust:
-    * https://github.com/jonathandturner/rls
-    * https://github.com/jonathandturner/rls_vscode
-    * https://github.com/RustDT/RustLSP