You cannot select more than 25 topics
Topics must start with a letter or number, can include dashes ('-') and can be up to 35 characters long.
72 lines
1.8 KiB
Plaintext
72 lines
1.8 KiB
Plaintext
import Lean
|
|
import GameServer.EnvExtensions
|
|
|
|
|
|
open Lean
|
|
|
|
structure GameServerState :=
|
|
(env : Lean.Environment)
|
|
(game : Name)
|
|
|
|
abbrev GameServerM := StateT GameServerState Server.Watchdog.ServerM
|
|
|
|
instance : MonadEnv GameServerM := {
|
|
getEnv := do return (← get).env
|
|
modifyEnv := fun f => do
|
|
let s ← get
|
|
set {s with env := f s.env}
|
|
}
|
|
|
|
namespace Game
|
|
open Server
|
|
open Watchdog
|
|
open Lsp
|
|
open JsonRpc
|
|
open IO
|
|
|
|
def getGame (game : Name): GameServerM Game := do
|
|
let some game ← getGame? game
|
|
| throwServerError "Game not found"
|
|
return game
|
|
|
|
structure LevelInfo where
|
|
index : Nat
|
|
title : String
|
|
tactics: Array TacticDocEntry
|
|
lemmas: Array LemmaDocEntry
|
|
introduction : String
|
|
deriving ToJson
|
|
|
|
structure LoadLevelParams where
|
|
world : Name
|
|
level : Nat
|
|
deriving ToJson, FromJson
|
|
|
|
partial def handleServerEvent (ev : ServerEvent) : GameServerM Bool := do
|
|
match ev with
|
|
| ServerEvent.clientMsg msg =>
|
|
match msg with
|
|
| Message.request id "info" _ =>
|
|
let s ← get
|
|
let c ← read
|
|
c.hOut.writeLspResponse ⟨id, (← getGame s.game)⟩
|
|
return true
|
|
| Message.request id "loadLevel" params =>
|
|
let p ← parseParams LoadLevelParams (toJson params)
|
|
let s ← get
|
|
let c ← read
|
|
let some lvl ← getLevel? {game := s.game, world := p.world, level := p.level}
|
|
| throwServerError s!"Level not found {(← getGame s.game).name} {p.world} {p.level}"
|
|
let levelInfo : LevelInfo :=
|
|
{ index := lvl.index,
|
|
title := lvl.title,
|
|
tactics := lvl.tactics,
|
|
lemmas := lvl.lemmas,
|
|
introduction := lvl.introduction }
|
|
c.hOut.writeLspResponse ⟨id, ToJson.toJson levelInfo⟩
|
|
return true
|
|
| _ => return false
|
|
| _ => return false
|
|
|
|
end Game
|