import LSpec import Pantograph.Serial import Pantograph.Environment import Test.Common namespace Pantograph.Test.Environment open Pantograph open Lean deriving instance DecidableEq, Repr for Protocol.InductInfo deriving instance DecidableEq, Repr for Protocol.ConstructorInfo deriving instance DecidableEq, Repr for Protocol.RecursorInfo deriving instance DecidableEq, Repr for Protocol.EnvInspectResult def test_symbol_visibility (env: Environment): IO LSpec.TestSeq := do let entries: List (Name × Bool) := [ ("Nat.add_comm".toName, false), ("Lean.Name".toName, true) ] let suite := entries.foldl (λ suites (symbol, target) => let constant := env.constants.find! symbol let test := LSpec.check symbol.toString ((Environment.is_symbol_unsafe_or_internal symbol constant) == target) LSpec.TestSeq.append suites test) LSpec.TestSeq.done return suite inductive ConstantCat where | induct (info: Protocol.InductInfo) | ctor (info: Protocol.ConstructorInfo) | recursor (info: Protocol.RecursorInfo) def test_inspect (env: Environment): IO LSpec.TestSeq := do let testCases: List (String × ConstantCat) := [ ("Or", ConstantCat.induct { numParams := 2, numIndices := 0, all := #["Or"], ctors := #["Or.inl", "Or.inr"], }), ("Except.ok", ConstantCat.ctor { induct := "Except", cidx := 1, numParams := 2, numFields := 1, }), ("Eq.rec", ConstantCat.recursor { all := #["Eq"], numParams := 2, numIndices := 1, numMotives := 1, numMinors := 1, k := true, }), ("ForM.rec", ConstantCat.recursor { all := #["ForM"], numParams := 3, numIndices := 0, numMotives := 1, numMinors := 1, k := false, }) ] let inner: CoreM LSpec.TestSeq := do testCases.foldlM (λ acc (name, cat) => do let args: Protocol.EnvInspect := { name := name } let result ← match ← Environment.inspect args (options := {}) with | .ok result => pure $ result | .error e => panic! s!"Error: {e.desc}" let p := match cat with | .induct info => LSpec.test name (result.inductInfo? == .some info) | .ctor info => LSpec.test name (result.constructorInfo? == .some info) | .recursor info => LSpec.test name (result.recursorInfo? == .some info) return LSpec.TestSeq.append acc p ) LSpec.TestSeq.done runCoreMSeq env inner def suite: IO LSpec.TestSeq := do let env: Environment ← importModules (imports := #[`Init]) --(imports := #["Prelude"].map (λ str => { module := str.toName, runtimeOnly := false })) (opts := {}) (trustLevel := 1) return LSpec.group "Environment" $ (LSpec.group "Symbol visibility" (← test_symbol_visibility env)) ++ (LSpec.group "Inspect" (← test_inspect env)) end Pantograph.Test.Environment