File tree Expand file tree Collapse file tree 2 files changed +2
-1
lines changed
Expand file tree Collapse file tree 2 files changed +2
-1
lines changed Original file line number Diff line number Diff line change @@ -117,7 +117,7 @@ def processParam (params : Grind.Params)
117117 throwError "invalid use of `intro` modifier, `{.ofConstName declName}` is not an inductive predicate"
118118 | .inj =>
119119 let thm ← Grind.mkInjectiveTheorem declName
120- params := { params with inj := params.inj.insert thm }
120+ params := { params with extraInj := params.extraInj.push thm }
121121 | .ext =>
122122 throwError "`[grind ext]` cannot be set using parameters"
123123 | .infer =>
Original file line number Diff line number Diff line change @@ -35,6 +35,7 @@ structure Params where
3535 symPrios : SymbolPriorities := {}
3636 casesTypes : CasesTypes := {}
3737 extra : PArray EMatchTheorem := {}
38+ extraInj : PArray InjectiveTheorem := {}
3839 norm : Simp.Context
3940 normProcs : Array Simprocs
4041 anchorRefs? : Option (Array AnchorRef) := none
You can’t perform that action at this time.
0 commit comments