Skip to content

Commit

Permalink
add info
Browse files Browse the repository at this point in the history
  • Loading branch information
gebner committed Apr 12, 2023
1 parent 5c72719 commit 37c0847
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/Tactic/Eqns.lean
Original file line number Diff line number Diff line change
Expand Up @@ -27,7 +27,7 @@ theorem transpose_const {m n} (c : ℕ) :
rw [transpose]
```
-/
open Lean
open Lean Elab

syntax (name := eqns) "eqns" ident* : attr

Expand All @@ -37,7 +37,7 @@ initialize eqnsAttribute : NameMapExtension (Array Name) ←
descr := "Overrides the equation lemmas for a declation to the provided list"
add := fun
| _, `(attr| eqns $[$names]*) =>
names.mapM resolveGlobalConstNoOverload
names.mapM resolveGlobalConstNoOverloadWithInfo
| _, _ => Lean.Elab.throwUnsupportedSyntax }

initialize Lean.Meta.registerGetEqnsFn (fun name => do
Expand Down

0 comments on commit 37c0847

Please sign in to comment.