Skip to content

Commit

Permalink
chore: move to v4.8.0-rc1
Browse files Browse the repository at this point in the history
  • Loading branch information
semorrison committed May 2, 2024
1 parent bed4e79 commit 89bc5a1
Show file tree
Hide file tree
Showing 6 changed files with 10 additions and 10 deletions.
4 changes: 2 additions & 2 deletions ProofWidgets/Data/Html.lean
Original file line number Diff line number Diff line change
Expand Up @@ -156,14 +156,14 @@ partial def delabHtmlElement' : DelabM (TSyntax `jsxElement) := do
let_expr Html.element tag _attrs _children := ← getExpr | failure

let .lit (.strVal s) := tag | failure
let tag ← withNaryArg 0 <| annotateTermLikeInfo <| mkIdent s
let tag ← withNaryArg 0 <| annotateTermLikeInfo <| mkIdent <| .mkSimple s

let attrs ← withNaryArg 1 <|
try
delabArrayLiteral <| withAnnotateTermLikeInfo do
let_expr Prod.mk _ _ a _ := ← getExpr | failure
let .lit (.strVal a) := a | failure
let attr ← withNaryArg 2 <| annotateTermLikeInfo <| mkIdent a
let attr ← withNaryArg 2 <| annotateTermLikeInfo <| mkIdent <| .mkSimple a
withNaryArg 3 do
let v ← getExpr
-- If the attribute's value is a string literal,
Expand Down
2 changes: 1 addition & 1 deletion ProofWidgets/Demos/Euclidean.lean
Original file line number Diff line number Diff line change
Expand Up @@ -245,7 +245,7 @@ def EuclideanConstructions.rpc (props : PanelWidgetProps) : RequestM (RequestTas
-- Find which hypotheses are selected.
let selectedHyps ← props.selectedLocations.filterMapM fun
| ⟨mv, .hyp fv⟩ | ⟨mv, .hypType fv _⟩ =>
return if mv == g.mvarId then some (← fv.getDecl) else none
if mv == g.mvarId then return some (← fv.getDecl) else return none
| _ =>
return none

Expand Down
2 changes: 1 addition & 1 deletion ProofWidgets/Demos/Venn.lean
Original file line number Diff line number Diff line change
Expand Up @@ -99,7 +99,7 @@ def VennDisplay.rpc (props : PanelWidgetProps) : RequestM (RequestTask Html) :=
Meta.withLCtx lctx md.localInstances do
let locs : Array LocalDecl ← props.selectedLocations.filterMapM fun
| ⟨mv, .hyp fv⟩ | ⟨mv, .hypType fv _⟩ =>
return if mv == g.mvarId then some (← fv.getDecl) else none
if mv == g.mvarId then return some (← fv.getDecl) else return none
| _ => return none
match ← isSetGoal? locs with
| some html => return html
Expand Down
4 changes: 2 additions & 2 deletions lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -4,10 +4,10 @@
[{"url": "https://github.com/leanprover/std4",
"type": "git",
"subDir": null,
"rev": "32983874c1b897d78f20d620fe92fc8fd3f06c3a",
"rev": "9fab3b45b6def355de20550141354cea24396224",
"name": "std",
"manifestFile": "lake-manifest.json",
"inputRev": "v4.7.0",
"inputRev": "nightly-testing",
"inherited": false,
"configFile": "lakefile.lean"}],
"name": "proofwidgets",
Expand Down
6 changes: 3 additions & 3 deletions lakefile.lean
Original file line number Diff line number Diff line change
Expand Up @@ -10,7 +10,7 @@ lean_lib ProofWidgets
lean_lib ProofWidgets.Demos where
globs := #[.submodules `ProofWidgets.Demos]

require std from git "https://github.com/leanprover/std4" @ "v4.7.0"
require std from git "https://github.com/leanprover/std4" @ "main"

def npmCmd : String :=
if Platform.isWindows then "npm.cmd" else "npm"
Expand All @@ -32,7 +32,7 @@ target widgetPackageLock : FilePath := do
Rebuilds whenever the `.tsx` source, or any part of the build configuration, has changed. -/
def widgetTsxTarget (pkg : NPackage _package.name) (nodeModulesMutex : IO.Mutex Bool)
(tsxName : String) (deps : Array (BuildJob FilePath)) (isDev : Bool) :
IndexBuildM (BuildJob FilePath) := do
FetchM (BuildJob FilePath) := do
let jsFile := pkg.buildDir / "js" / s!"{tsxName}.js"
buildFileAfterDepArray jsFile deps fun _srcFile => do
/-
Expand Down Expand Up @@ -67,7 +67,7 @@ def widgetTsxTarget (pkg : NPackage _package.name) (nodeModulesMutex : IO.Mutex

/-- Target to build all TypeScript widget modules that match `widget/src/*.tsx`. -/
def widgetJsAllTarget (pkg : NPackage _package.name) (isDev : Bool) :
IndexBuildM (BuildJob (Array FilePath)) := do
FetchM (BuildJob (Array FilePath)) := do
let fs ← (widgetDir / "src").readDir
let tsxs : Array FilePath := fs.filterMap fun f =>
let p := f.path; if let some "tsx" := p.extension then some p else none
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.7.0
leanprover/lean4:v4.8.0-rc1

0 comments on commit 89bc5a1

Please sign in to comment.