Documentation
Lean
.
Elab
.
PreDefinition
.
Structural
.
Eqns
Search
return to top
source
Imports
Lean.Meta.Eqns
Lean.Elab.PreDefinition.Basic
Lean.Elab.PreDefinition.Eqns
Lean.Meta.Tactic.Apply
Lean.Meta.Tactic.Split
Lean.Elab.PreDefinition.Structural.Basic
Lean.Meta.Tactic.Simp.Main
Imported by
Lean
.
Elab
.
Structural
.
EqnInfo
Lean
.
Elab
.
Structural
.
instInhabitedEqnInfo
Lean
.
Elab
.
Structural
.
mkEqns
Lean
.
Elab
.
Structural
.
eqnInfoExt
Lean
.
Elab
.
Structural
.
registerEqnsInfo
Lean
.
Elab
.
Structural
.
getEqnsFor?
Lean
.
Elab
.
Structural
.
getUnfoldFor?
Lean
.
Elab
.
Structural
.
getStructuralRecArgPosImp?
source
structure
Lean
.
Elab
.
Structural
.
EqnInfo
extends
Lean.Elab.Eqns.EqnInfoCore
:
Type
declName
:
Name
levelParams
:
List
Name
type
:
Expr
value
:
Expr
recArgPos :
Nat
declNames :
Array
Name
numFixed :
Nat
Instances For
source
instance
Lean
.
Elab
.
Structural
.
instInhabitedEqnInfo
:
Inhabited
EqnInfo
Equations
Lean.Elab.Structural.instInhabitedEqnInfo
=
{
default
:=
{
toEqnInfoCore
:=
default
,
recArgPos
:=
default
,
declNames
:=
default
,
numFixed
:=
default
}
}
source
def
Lean
.
Elab
.
Structural
.
mkEqns
(info :
EqnInfo
)
:
MetaM
(
Array
Name
)
Equations
One or more equations did not get rendered due to their size.
Instances For
source
opaque
Lean
.
Elab
.
Structural
.
eqnInfoExt
:
MapDeclarationExtension
EqnInfo
source
def
Lean
.
Elab
.
Structural
.
registerEqnsInfo
(preDef :
PreDefinition
)
(declNames :
Array
Name
)
(recArgPos numFixed :
Nat
)
:
CoreM
Unit
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Elab
.
Structural
.
getEqnsFor?
(declName :
Name
)
:
MetaM
(
Option
(
Array
Name
)
)
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Elab
.
Structural
.
getUnfoldFor?
(declName :
Name
)
:
MetaM
(
Option
Name
)
Equations
One or more equations did not get rendered due to their size.
Instances For
source
@[export lean_get_structural_rec_arg_pos]
def
Lean
.
Elab
.
Structural
.
getStructuralRecArgPosImp?
(declName :
Name
)
:
CoreM
(
Option
Nat
)
Equations
One or more equations did not get rendered due to their size.
Instances For