diff --git a/Mathlib/Tactic/CC/Addition.lean b/Mathlib/Tactic/CC/Addition.lean index 402aa77e105b8..2b3349c44376a 100644 --- a/Mathlib/Tactic/CC/Addition.lean +++ b/Mathlib/Tactic/CC/Addition.lean @@ -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 diff --git a/Mathlib/Tactic/FunProp/RefinedDiscrTree.lean b/Mathlib/Tactic/FunProp/RefinedDiscrTree.lean index 876dc3a14dc35..1f6cdbcd5f5f6 100644 --- a/Mathlib/Tactic/FunProp/RefinedDiscrTree.lean +++ b/Mathlib/Tactic/FunProp/RefinedDiscrTree.lean @@ -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 diff --git a/lake-manifest.json b/lake-manifest.json index d965eb5cdb0eb..56aad3d6219de 100644 --- a/lake-manifest.json +++ b/lake-manifest.json @@ -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", @@ -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", diff --git a/lakefile.lean b/lakefile.lean index 0fb8c72d4767f..f32677f0edb1b 100644 --- a/lakefile.lean +++ b/lakefile.lean @@ -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"