Skip to content

Commit

Permalink
chore: bump to v4.15.0-rc1 (#61)
Browse files Browse the repository at this point in the history
* chore: bump to v4.15.0-rc1

* fix InfoTree.lean (cf. leanprover/lean4#5835)

* fix: workaround for Meta.Context.config private (#64)

---------

Co-authored-by: Bryan Gin-ge Chen <[email protected]>
Co-authored-by: L <[email protected]>
  • Loading branch information
3 people authored Jan 8, 2025
1 parent d7545ee commit 008cfbc
Show file tree
Hide file tree
Showing 6 changed files with 30 additions and 25 deletions.
18 changes: 11 additions & 7 deletions REPL/Lean/InfoTree.lean
Original file line number Diff line number Diff line change
Expand Up @@ -53,6 +53,7 @@ namespace Lean.Elab.Info
def kind : Info → String
| .ofTacticInfo _ => "TacticInfo"
| .ofTermInfo _ => "TermInfo"
| ofPartialTermInfo _ => "PartialTermInfo"
| .ofCommandInfo _ => "CommmandInfo"
| .ofMacroExpansionInfo _ => "MacroExpansionInfo"
| .ofOptionInfo _ => "OptionInfo"
Expand All @@ -63,11 +64,13 @@ def kind : Info → String
| .ofFVarAliasInfo _ => "FVarAliasInfo"
| .ofFieldRedeclInfo _ => "FieldRedeclInfo"
| .ofOmissionInfo _ => "OmissionInfo"
| .ofChoiceInfo _ => "ChoiceInfo"

/-- The `Syntax` for a `Lean.Elab.Info`, if there is one. -/
def stx? : Info → Option Syntax
| .ofTacticInfo info => info.stx
| .ofTermInfo info => info.stx
| ofPartialTermInfo info => info.stx
| .ofCommandInfo info => info.stx
| .ofMacroExpansionInfo info => info.stx
| .ofOptionInfo info => info.stx
Expand All @@ -78,6 +81,7 @@ def stx? : Info → Option Syntax
| .ofFVarAliasInfo _ => none
| .ofFieldRedeclInfo info => info.stx
| .ofOmissionInfo info => info.stx
| .ofChoiceInfo info => info.stx

/-- Is the `Syntax` for this `Lean.Elab.Info` original, or synthetic? -/
def isOriginal (i : Info) : Bool :=
Expand Down Expand Up @@ -214,13 +218,13 @@ def sorries (t : InfoTree) : List (ContextInfo × SorryType × Position × Posit

def tactics (t : InfoTree) : List (ContextInfo × Syntax × List MVarId × Position × Position × Array Name) :=
-- HACK: creating a child ngen
t.findTacticNodes.map fun ⟨i, ctx⟩ =>
let range := stxRange ctx.fileMap i.stx
( { ctx with mctx := i.mctxBefore, ngen := ctx.ngen.mkChild.1 },
i.stx,
i.goalsBefore,
range.fst,
range.snd,
t.findTacticNodes.map fun ⟨i, ctx⟩ =>
let range := stxRange ctx.fileMap i.stx
( { ctx with mctx := i.mctxBefore, ngen := ctx.ngen.mkChild.1 },
i.stx,
i.goalsBefore,
range.fst,
range.snd,
i.getUsedConstantsAsSet.toArray )


Expand Down
3 changes: 2 additions & 1 deletion REPL/Snapshots.lean
Original file line number Diff line number Diff line change
Expand Up @@ -259,13 +259,14 @@ When pickling the `Environment`, we do so relative to its imports.
def pickle (p : ProofSnapshot) (path : FilePath) : IO Unit := do
let env := p.coreState.env
let p' := { p with coreState := { p.coreState with env := ← mkEmptyEnvironment }}
let (cfg, _) ← Lean.Meta.getConfig.toIO p'.coreContext p'.coreState p'.metaContext p'.metaState
_root_.pickle path
(env.header.imports,
env.constants.map₂,
({ p'.coreState with } : CompactableCoreState),
p'.coreContext,
p'.metaState,
({ p'.metaContext with } : CompactableMetaContext),
({ p'.metaContext with config := cfg } : CompactableMetaContext),
p'.termState,
({ p'.termContext with } : CompactableTermContext),
p'.tacticState,
Expand Down
2 changes: 1 addition & 1 deletion lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:v4.14.0
leanprover/lean4:v4.15.0-rc1
28 changes: 14 additions & 14 deletions test/Mathlib/lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -5,20 +5,20 @@
"type": "git",
"subDir": null,
"scope": "",
"rev": "4bbdccd9c5f862bf90ff12f0a9e2c8be032b9a84",
"rev": "41ff1f7899c971f91362710d4444e338b8acd644",
"name": "mathlib",
"manifestFile": "lake-manifest.json",
"inputRev": "v4.14.0",
"inputRev": "v4.15.0-rc1",
"inherited": false,
"configFile": "lakefile.lean"},
{"url": "https://github.com/leanprover-community/plausible",
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "42dc02bdbc5d0c2f395718462a76c3d87318f7fa",
"rev": "8e5cb8d424df462f84997dd68af6f40e347c3e35",
"name": "plausible",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
"inputRev": "v4.15.0-rc1",
"inherited": true,
"configFile": "lakefile.toml"},
{"url": "https://github.com/leanprover-community/LeanSearchClient",
Expand All @@ -35,47 +35,47 @@
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "519e509a28864af5bed98033dd33b95cf08e9aa7",
"rev": "ed3b856bd8893ade75cafe13e8544d4c2660f377",
"name": "importGraph",
"manifestFile": "lake-manifest.json",
"inputRev": "v4.14.0",
"inputRev": "v4.15.0-rc1",
"inherited": true,
"configFile": "lakefile.toml"},
{"url": "https://github.com/leanprover-community/ProofWidgets4",
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "68280daef58803f68368eb2e53046dabcd270c9d",
"rev": "2b000e02d50394af68cfb4770a291113d94801b5",
"name": "proofwidgets",
"manifestFile": "lake-manifest.json",
"inputRev": "v0.0.47",
"inputRev": "v0.0.48",
"inherited": true,
"configFile": "lakefile.lean"},
{"url": "https://github.com/leanprover-community/aesop",
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "5a0ec8588855265ade536f35bcdcf0fb24fd6030",
"rev": "8b6048aa0a4a4b6bcf83597802d8dee734e64b7e",
"name": "aesop",
"manifestFile": "lake-manifest.json",
"inputRev": "v4.14.0",
"inputRev": "v4.15.0-rc1",
"inherited": true,
"configFile": "lakefile.toml"},
{"url": "https://github.com/leanprover-community/quote4",
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "303b23fbcea94ac4f96e590c1cad6618fd4f5f41",
"rev": "ad942fdf0b15c38bface6acbb01d63855a2519ac",
"name": "Qq",
"manifestFile": "lake-manifest.json",
"inputRev": "master",
"inputRev": "v4.14.0",
"inherited": true,
"configFile": "lakefile.lean"},
{"url": "https://github.com/leanprover-community/batteries",
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "8d6c853f11a5172efa0e96b9f2be1a83d861cdd9",
"rev": "7805acf1864ba1a2e359f86a8f092ccf1438ad83",
"name": "batteries",
"manifestFile": "lake-manifest.json",
"inputRev": "v4.14.0",
Expand All @@ -85,7 +85,7 @@
"type": "git",
"subDir": null,
"scope": "leanprover",
"rev": "726b3c9ad13acca724d4651f14afc4804a7b0e4d",
"rev": "0c8ea32a15a4f74143e4e1e107ba2c412adb90fd",
"name": "Cli",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
Expand Down
2 changes: 1 addition & 1 deletion test/Mathlib/lakefile.toml
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ defaultTargets = ["ReplMathlibTests"]
[[require]]
name = "mathlib"
git = "https://github.com/leanprover-community/mathlib4"
rev = "v4.14.0"
rev = "v4.15.0-rc1"

[[lean_lib]]
name = "ReplMathlibTests"
Expand Down
2 changes: 1 addition & 1 deletion test/Mathlib/lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:v4.14.0
leanprover/lean4:v4.15.0-rc1

0 comments on commit 008cfbc

Please sign in to comment.