Equations
- Lean.Meta.AC.instInhabitedPreContext = { default := { id := default, op := default, assoc := default, comm := default, idem := default } }
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.
@[matchPattern]
def
Lean.Meta.AC.bin
{x₁ : Lean.Expr.Data}
{x₂ : Lean.Expr.Data}
(op : Lean.Expr)
(l : Lean.Expr)
(r : Lean.Expr)
:
Equations
- Lean.Meta.AC.bin op l r = Lean.Expr.app (Lean.Expr.app op l x₁) r x₂
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Meta.AC.toACExpr.toACExpr varMap (Lean.Meta.AC.PreExpr.op l 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) = Lean.Data.AC.Expr.var (varMap x)
def
Lean.Meta.AC.buildNormProof
(preContext : Lean.Meta.AC.PreContext)
(l : Lean.Expr)
(r : Lean.Expr)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Meta.AC.buildNormProof.mkContext
(preContext : Lean.Meta.AC.PreContext)
(α : Lean.Expr)
(u : Lean.Level)
(vars : Array Lean.Expr)
:
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Meta.AC.buildNormProof.convert (Lean.Data.AC.Expr.op l 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) = Lean.mkApp (Lean.mkConst `Lean.Data.AC.Expr.var) (Lean.mkNatLit x)
def
Lean.Meta.AC.buildNormProof.convertTarget
(preContext : Lean.Meta.AC.PreContext)
(vars : Array Lean.Expr)
:
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) = Array.getOp vars x
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.Meta.AC.ac_refl_tactic x = do let goal ← Lean.Elab.Tactic.getMainGoal liftM (Lean.Meta.AC.rewriteUnnormalized goal)