Documentation
Lean
.
Meta
.
Tactic
.
Grind
.
Arith
.
Linear
.
Internalize
Search
return to top
source
Imports
Lean.Meta.Tactic.Grind.Simp
Lean.Meta.Tactic.Grind.Arith.CommRing.Reify
Lean.Meta.Tactic.Grind.Arith.Linear.Reify
Lean.Meta.Tactic.Grind.Arith.Linear.StructId
Imported by
Lean
.
Meta
.
Grind
.
Arith
.
Linear
.
markVars
Lean
.
Meta
.
Grind
.
Arith
.
Linear
.
internalize
source
def
Lean
.
Meta
.
Grind
.
Arith
.
Linear
.
markVars
(
e
:
Expr
)
:
LinearM
Unit
Equations
Lean.Meta.Grind.Arith.Linear.markVars
e
=
discard
(
Lean.Meta.Grind.Arith.Linear.reify?
e
true
)
Instances For
source
def
Lean
.
Meta
.
Grind
.
Arith
.
Linear
.
internalize
(
e
:
Expr
)
(
parent?
:
Option
Expr
)
:
GoalM
Unit
Equations
One or more equations did not get rendered due to their size.
Instances For