@[reducible, inline]
Equations
Instances For
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.
Instances For
Equations
- One or more equations did not get rendered due to their size.
- Lean.Meta.AC.toACExpr.toPreExpr op x✝ = do modify fun (vars : Lean.ExprSet) => Std.HashSet.insert vars x✝ pure (Lean.Meta.AC.PreExpr.var x✝)
Instances For
Equations
- Lean.Meta.AC.toACExpr.toACExpr varMap (l.op r) = Lean.Data.AC.Expr.op (Lean.Meta.AC.toACExpr.toACExpr varMap l) (Lean.Meta.AC.toACExpr.toACExpr varMap r)
- Lean.Meta.AC.toACExpr.toACExpr varMap (Lean.Meta.AC.PreExpr.var x_1) = Lean.Data.AC.Expr.var (varMap x_1)
Instances For
def
Lean.Meta.AC.abstractAtoms
(preContext : PreContext)
(atoms : Array Expr)
(k : Array (Expr × Option Expr) → MetaM Expr)
 :
In order to prevent the kernel trying to reduce the atoms of the expression, we abstract the proof
over them. But ac_rfl proofs are not completely abstract in the value of the atoms – it recognizes
neutral elements. So we have to abstract over these proofs as well.
Equations
- Lean.Meta.AC.abstractAtoms preContext atoms k = do let α ← Lean.Meta.inferType atoms[0]! let u ← Lean.Meta.getLevel α Lean.Meta.AC.abstractAtoms.go preContext atoms k α u 0 #[] #[] #[]
Instances For
@[irreducible]
def
Lean.Meta.AC.abstractAtoms.go
(preContext : PreContext)
(atoms : Array Expr)
(k : Array (Expr × Option Expr) → MetaM Expr)
(α : Expr)
(u : Level)
(i : Nat)
(acc : Array (Expr × Option Expr))
(vars args : Array Expr)
 :
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
- Lean.Meta.AC.buildNormProof.convert (l.op r) = Lean.mkApp2 (Lean.mkConst `Lean.Data.AC.Expr.op) (Lean.Meta.AC.buildNormProof.convert l) (Lean.Meta.AC.buildNormProof.convert r)
- Lean.Meta.AC.buildNormProof.convert (Lean.Data.AC.Expr.var x_1) = Lean.mkApp (Lean.mkConst `Lean.Data.AC.Expr.var) (Lean.mkNatLit x_1)
Instances For
Equations
- One or more equations did not get rendered due to their size.
- Lean.Meta.AC.buildNormProof.convertTarget preContext vars (Lean.Data.AC.Expr.var x_1) = vars[x_1]!
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
- Lean.Meta.AC.rewriteUnnormalizedRefl goal = do let __do_lift ← Lean.Meta.AC.rewriteUnnormalized goal __do_lift.refl
Instances For
Equations
- Lean.Meta.AC.acRflTactic x✝ = do let goal ← Lean.Elab.Tactic.getMainGoal goal.withContext (liftM (Lean.Meta.AC.rewriteUnnormalizedRefl goal))
Instances For
Implementation of the ac_nf tactic when operating on the main goal.
Equations
- Lean.Meta.AC.acNfTargetTactic = Lean.Elab.Tactic.liftMetaTactic1 fun (goal : Lean.MVarId) => do let a ← Lean.Meta.AC.rewriteUnnormalized goal pure (some a)
Instances For
Implementation of the ac_nf tactic when operating on a hypothesis.
Equations
- Lean.Meta.AC.acNfHypTactic fvarId = Lean.Elab.Tactic.liftMetaTactic1 fun (goal : Lean.MVarId) => Lean.Meta.AC.acNfHypMeta goal fvarId
Instances For
Equations
- One or more equations did not get rendered due to their size.