Skip to content

Commit 91bc2ab

Browse files
digama0gebner
andcommitted
chore: update std 12-05 (#863)
Co-authored-by: Gabriel Ebner <gebner@gebner.org>
1 parent 0510151 commit 91bc2ab

File tree

3 files changed

+4
-11
lines changed

3 files changed

+4
-11
lines changed

Mathlib/Lean/Expr/Basic.lean

Lines changed: 1 addition & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -6,6 +6,7 @@ Floris van Doorn, E.W.Ayers, Arthur Paulino
66
-/
77
import Lean
88
import Mathlib.Util.MapsTo
9+
import Std.Lean.Expr
910
import Std.Data.List.Basic
1011

1112
/-!
@@ -264,14 +265,6 @@ def addLocalVarInfoForBinderIdent (fvar : Expr) : TSyntax ``binderIdent → Term
264265
| `(binderIdent| $n:ident) => Elab.Term.addLocalVarInfo n fvar
265266
| tk => Elab.Term.addLocalVarInfo (Unhygienic.run `(_%$tk)) fvar
266267

267-
/-- Converts an `Expr` into a `Syntax`, by creating a fresh metavariable
268-
assigned to the expr and returning a named metavariable syntax `?a`. -/
269-
def toSyntax (e : Expr) : TermElabM Syntax.Term := withFreshMacroScope do
270-
let stx ← `(?a)
271-
let mvar ← elabTermEnsuringType stx (← Meta.inferType e)
272-
mvar.mvarId!.assign e
273-
pure stx
274-
275268
end Expr
276269

277270
end Lean

Mathlib/Order/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -655,7 +655,7 @@ variable [Preorder α] [Nonempty β] {a b : α}
655655

656656
@[simp] lemma const_le_const : const β a ≤ const β b ↔ a ≤ b := by simp [Pi.le_def]
657657
@[simp] lemma const_lt_const : const β a < const β b ↔ a < b := by
658-
simpa [Pi.lt_def] using le_of_lt (α := _)
658+
simpa [Pi.lt_def] using le_of_lt (α := α)
659659

660660
end Function
661661

lake-manifest.json

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -34,7 +34,7 @@
3434
{"git":
3535
{"url": "https://github.com/JLimperg/aesop",
3636
"subDir?": null,
37-
"rev": "70c59fcfc63de90786d59222c32468dab87964c5",
37+
"rev": "61004154b4a8f7aec6224745f4fbddeda5795e97",
3838
"name": "aesop",
3939
"inputRev?": "master"}},
4040
{"git":
@@ -52,6 +52,6 @@
5252
{"git":
5353
{"url": "https://github.com/leanprover/std4",
5454
"subDir?": null,
55-
"rev": "42bb39d34ec7dcb07580458efa4a7936bd5192b7",
55+
"rev": "cad19f171ad4aebe091e6deeb9a43a14521bfbfe",
5656
"name": "std",
5757
"inputRev?": "main"}}]}

0 commit comments

Comments
 (0)