Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Elab.Tactic.isCheckpointableTactic arg = let kind := Lean.Syntax.getKind arg; pure (kind == `Lean.Parser.Tactic.save)
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
partial def
Lean.Elab.Tactic.addCheckpoints.go
(args : Array Lean.Syntax)
(i : Nat)
(acc : Array Lean.Syntax)
(result : Array Lean.Syntax)
:
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Elab.Tactic.evalRotateLeft stx = let n := Lean.Elab.Tactic.getOptRotation (Lean.Syntax.getOp stx 1); do let a ← Lean.Elab.Tactic.getGoals Lean.Elab.Tactic.setGoals (List.rotateLeft a n)
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Elab.Tactic.evalAssumption x = Lean.Elab.Tactic.liftMetaTactic fun mvarId => do Lean.Meta.assumption mvarId pure []
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Elab.Tactic.evalRefl x = Lean.Elab.Tactic.liftMetaTactic fun mvarId => do Lean.Meta.refl mvarId pure []
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Tactic.forEachVar
(hs : Array Lean.Syntax)
(tac : Lean.MVarId → Lean.FVarId → Lean.MetaM Lean.MVarId)
:
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Elab.Tactic.evalSubstVars x = Lean.Elab.Tactic.liftMetaTactic fun mvarId => do let a ← Lean.Meta.substVars mvarId pure [a]
def
Lean.Elab.Tactic.renameInaccessibles
(mvarId : Lean.MVarId)
(hs : Lean.TSyntaxArray `Lean.binderIdent)
:
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Elab.Tactic.evalSleep stx = match Lean.Syntax.isNatLit? (Lean.Syntax.getOp stx 1) with | none => Lean.Elab.throwIllFormedSyntax | some ms => liftM (IO.sleep (Nat.toUInt32 ms))