Propagator for dependent forall terms
forall (h : p), q[h] where p is a proposition.
Equations
- One or more equations did not get rendered due to their size.
- Lean.Meta.Grind.propagateForallPropUp e = pure ()
Instances For
Given a proof of an EMatchTheorem, returns true, if there are no
anchor references restricting the search, or there is an anchor
references ref s.t. ref matches proof.
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.Grind.propagateForallPropDown e = pure ()
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Applies the following rewriting rules:
Grind.imp_true_eqGrind.imp_false_eqGrind.forall_imp_eq_orGrind.true_imp_eqGrind.false_imp_eqGrind.imp_self_eqforall_trueforall_falseGrind.forall_or_forallGrind.forall_forall_orGrind.forall_and
Equations
- One or more equations did not get rendered due to their size.
- Lean.Meta.Grind.simpForall e = pure Lean.Meta.Simp.Step.continue
Instances For
Applies the following rewriting rules:
Grind.exists_orGrind.exists_and_leftGrind.exists_and_rightGrind.exists_propGrind.exists_const
Equations
- One or more equations did not get rendered due to their size.