Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.Script.TacticBuilder.apply
(mvarId : Lean.MVarId)
(e : Lean.Expr)
(md : Lean.Meta.TransparencyMode)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.Script.TacticBuilder.exactFVar
(goal : Lean.MVarId)
(fvarId : Lean.FVarId)
(md : Lean.Meta.TransparencyMode)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.Script.TacticBuilder.replace
(preGoal : Lean.MVarId)
(postGoal : Lean.MVarId)
(fvarId : Lean.FVarId)
(type : Lean.Expr)
(proof : Lean.Expr)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.Script.TacticBuilder.assertHypothesis
(goal : Lean.MVarId)
(h : Lean.Meta.Hypothesis)
(md : Lean.Meta.TransparencyMode)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.Script.TacticBuilder.cases
(goal : Lean.MVarId)
(e : Lean.Expr)
(ctorNames : Array Aesop.CtorNames)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.Script.TacticBuilder.obtain
(goal : Lean.MVarId)
(e : Lean.Expr)
(ctorNames : Aesop.CtorNames)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.Script.TacticBuilder.casesOrObtain
(goal : Lean.MVarId)
(e : Lean.Expr)
(ctorNames : Array Aesop.CtorNames)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.Script.TacticBuilder.renameInaccessibleFVars
(postGoal : Lean.MVarId)
(renamedFVars : Array Lean.FVarId)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.Script.TacticBuilder.unfoldAt
(goal : Lean.MVarId)
(fvarId : Lean.FVarId)
(usedDecls : Array Lean.Name)
(aesopUnfold : Bool)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.Script.TacticBuilder.extN.mkPat
(fvarId : Lean.FVarId)
:
Lean.MetaM (Lean.TSyntax `rintroPat)
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.Script.TacticBuilder.simpAllOrSimpAtStarOnly
(simpAll : Bool)
(inGoal : Lean.MVarId)
(configStx? : Option Lean.Term)
(usedTheorems : Lean.Meta.Simp.UsedSimps)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.Script.TacticBuilder.simpAllOrSimpAtStar
(simpAll : Bool)
(inGoal : Lean.MVarId)
(configStx? : Option Lean.Term)
(usedTheorems : Lean.Meta.Simp.UsedSimps)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.Script.TacticBuilder.intros
(postGoal : Lean.MVarId)
(newFVarIds : Array Lean.FVarId)
(md : Lean.Meta.TransparencyMode)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.assertHypothesisS
(goal : Lean.MVarId)
(h : Lean.Meta.Hypothesis)
(md : Lean.Meta.TransparencyMode)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.assertHypothesisS.tacticBuilder
(goal : Lean.MVarId)
(h : Lean.Meta.Hypothesis)
(md : Lean.Meta.TransparencyMode)
:
Equations
- Aesop.assertHypothesisS.tacticBuilder goal h md x = Aesop.Script.TacticBuilder.assertHypothesis goal h md
Instances For
def
Aesop.applyS
(goal : Lean.MVarId)
(e : Lean.Expr)
(eStx? : Option Lean.Term)
(md : Lean.Meta.TransparencyMode)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.applyS.tacticBuilder
(goal : Lean.MVarId)
(e : Lean.Expr)
(eStx? : Option Lean.Term)
(md : Lean.Meta.TransparencyMode)
:
Equations
- Aesop.applyS.tacticBuilder goal e none md x = Aesop.Script.TacticBuilder.apply goal e md
- Aesop.applyS.tacticBuilder goal e (some cfg) md x = Aesop.Script.TacticBuilder.applyStx cfg md
Instances For
def
Aesop.replaceFVarS
(goal : Lean.MVarId)
(fvarId : Lean.FVarId)
(type : Lean.Expr)
(proof : Lean.Expr)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.replaceFVarS.tacticBuilder
(goal : Lean.MVarId)
(fvarId : Lean.FVarId)
(type : Lean.Expr)
(proof : Lean.Expr)
:
Equations
- Aesop.replaceFVarS.tacticBuilder goal fvarId type proof x = Aesop.Script.TacticBuilder.replace goal x.fst fvarId type proof
Instances For
Equations
- Aesop.clearS goal fvarId = Aesop.withScriptStep goal (fun (x : Lean.MVarId) => #[x]) (fun (x : Lean.MVarId) => true) (Aesop.clearS.tacticBuilder goal fvarId) (goal.clear fvarId)
Instances For
Equations
- Aesop.clearS.tacticBuilder goal fvarId x = Aesop.Script.TacticBuilder.clear goal #[fvarId]
Instances For
Equations
- Aesop.tryClearS goal fvarId = Aesop.withOptScriptStep goal (fun (x : Lean.MVarId) => #[x]) (Aesop.tryClearS.tacticBuilder goal fvarId) do let a ← goal.tryClear fvarId pure (some a)
Instances For
Equations
- Aesop.tryClearS.tacticBuilder goal fvarId x = Aesop.Script.TacticBuilder.clear goal #[fvarId]
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Aesop.tryClearManyS.tacticBuilder goal (g, fvarIds) = Aesop.Script.TacticBuilder.clear goal fvarIds
Instances For
def
Aesop.tryCasesS
(goal : Lean.MVarId)
(fvarId : Lean.FVarId)
(ctorNames : Array Aesop.CtorNames)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.tryCasesS.getUnusedCtorNames
(ctorNames : Array Aesop.CtorNames)
(lctx : Lean.LocalContext)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Aesop.renameInaccessibleFVarsS.tacticBuilder (g, fvarIds) = Aesop.Script.TacticBuilder.renameInaccessibleFVars g fvarIds
Instances For
def
Aesop.unfoldManyTargetS
(unfold? : Lean.Name → Option (Option Lean.Name))
(goal : Lean.MVarId)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.unfoldManyAtS
(unfold? : Lean.Name → Option (Option Lean.Name))
(goal : Lean.MVarId)
(fvarId : Lean.FVarId)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Aesop.introsS.tacticBuilder (g, fvarIds) = Aesop.Script.TacticBuilder.intros g fvarIds Lean.Meta.TransparencyMode.default
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Aesop.introsUnfoldingS.tacticBuilder md (g, fvarIds) = Aesop.Script.TacticBuilder.intros g fvarIds md
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.tryExactFVarS
(goal : Lean.MVarId)
(fvarId : Lean.FVarId)
(md : Lean.Meta.TransparencyMode)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Aesop.splitFirstHypothesisS?.tacticBuilder goal (fst, fvarId) = Aesop.Script.TacticBuilder.splitAt goal fvarId