def
Aesop.RuleTac.applyExpr'
(goal : Lean.MVarId)
(e : Lean.Expr)
(eStx : Lean.Term)
(pat? : Option Aesop.RulePattern)
(patInst : Aesop.RulePatternInstantiation)
(md : Lean.Meta.TransparencyMode)
 :
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.RuleTac.applyExpr
(goal : Lean.MVarId)
(e : Lean.Expr)
(eStx : Lean.Term)
(pat? : Option Aesop.RulePattern)
(patInsts : Lean.HashSet Aesop.RulePatternInstantiation)
(md : Lean.Meta.TransparencyMode)
 :
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.RuleTac.applyConst
(decl : Lean.Name)
(pat? : Option Aesop.RulePattern)
(md : Lean.Meta.TransparencyMode)
 :
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.RuleTac.applyTerm
(stx : Lean.Term)
(pat? : Option Aesop.RulePattern)
(md : Lean.Meta.TransparencyMode)
 :
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.RuleTac.apply
(t : Aesop.RuleTerm)
(pat? : Option Aesop.RulePattern)
(md : Lean.Meta.TransparencyMode)
 :
Equations
- Aesop.RuleTac.apply t pat? md = match t with | Aesop.RuleTerm.const decl => Aesop.RuleTac.applyConst decl pat? md | Aesop.RuleTerm.term tm => Aesop.RuleTac.applyTerm tm pat? md
Instances For
Equations
- One or more equations did not get rendered due to their size.