Equations
Equations
Equations
Equations
- Lean.Elab.Tactic.Do.Uses.zero.add x✝ = x✝
- x✝.add Lean.Elab.Tactic.Do.Uses.zero = x✝
- x✝¹.add x✝ = Lean.Elab.Tactic.Do.Uses.many
Instances For
Equations
Instances For
Equations
@[reducible, inline]
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Equations
- Lean.Elab.Tactic.Do.BVarUses.none.add b = b
- a.add Lean.Elab.Tactic.Do.BVarUses.none = a
- (Lean.Elab.Tactic.Do.BVarUses.some a_2).add (Lean.Elab.Tactic.Do.BVarUses.some b_2) = Lean.Elab.Tactic.Do.BVarUses.some (Vector.zipWith (fun (a b : Lean.Elab.Tactic.Do.Uses) => a + b) a_2 b_2)
Instances For
Equations
Equations
- Lean.Elab.Tactic.Do.addMData d (Lean.Expr.mdata d' e_2) = Lean.Expr.mdata (Lean.KVMap.mergeBy (fun (x : Lean.Name) (new x : Lean.DataValue) => new) d d') e_2
- Lean.Elab.Tactic.Do.addMData d e = Lean.Expr.mdata d e
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Elab.Tactic.Do.doNotDup u rhs elimTrivial = (u == Lean.Elab.Tactic.Do.Uses.many && !(elimTrivial && Lean.Elab.Tactic.Do.okToDup✝ rhs))