Skip to content

Commit

Permalink
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Nov 11, 2024
1 parent f27c375 commit b8f1ecb
Show file tree
Hide file tree
Showing 4 changed files with 6 additions and 6 deletions.
2 changes: 1 addition & 1 deletion Mathlib/Tactic/CC/Addition.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1748,7 +1748,7 @@ def propagateProjectionConstructor (p c : Expr) : CCM Unit := do
unless ← pureIsDefEq (← inferType (pArgs[mkidx]'h)) (← inferType c) do return
/- Create new projection application using c (e.g., `(x, y).fst`), and internalize it.
The internalizer will add the new equality. -/
let pArgs := pArgs.set mkidx, h⟩ c
let pArgs := pArgs.set mkidx c
let newP := mkAppN pFn pArgs
internalizeCore newP none
else
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Tactic/FunProp/RefinedDiscrTree.lean
Original file line number Diff line number Diff line change
Expand Up @@ -875,7 +875,7 @@ where
loop (i : Nat) : Array α :=
if h : i < vs.size then
if v == vs[i] then
vs.set ⟨i,h⟩ v
vs.set i v
else
loop (i+1)
else
Expand Down
6 changes: 3 additions & 3 deletions lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "d9e997fb60f8d4fcbf03270fbb696f7c87ee0e25",
"rev": "4fbc598626f02cae3d60708c04a09c311bb60369",
"name": "batteries",
"manifestFile": "lake-manifest.json",
"inputRev": "lean-pr-testing-5988",
Expand All @@ -25,10 +25,10 @@
"type": "git",
"subDir": null,
"scope": "leanprover-community",
"rev": "45d016d59cf45bcf8493a203e9564cfec5203d9b",
"rev": "fa36772c08508c85c9ba531a8865cdeb391631df",
"name": "aesop",
"manifestFile": "lake-manifest.json",
"inputRev": "master",
"inputRev": "lean-pr-testing-5988",
"inherited": false,
"configFile": "lakefile.toml"},
{"url": "https://github.com/leanprover-community/ProofWidgets4",
Expand Down
2 changes: 1 addition & 1 deletion lakefile.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,7 +9,7 @@ open Lake DSL

require "leanprover-community" / "batteries" @ git "lean-pr-testing-5988"
require "leanprover-community" / "Qq" @ git "master"
require "leanprover-community" / "aesop" @ git "master"
require "leanprover-community" / "aesop" @ git "lean-pr-testing-5988"
require "leanprover-community" / "proofwidgets" @ git "v0.0.46"
require "leanprover-community" / "importGraph" @ git "main"
require "leanprover-community" / "LeanSearchClient" @ git "main"
Expand Down

0 comments on commit b8f1ecb

Please sign in to comment.