Unfolds an appropriate PartialOrder
instance on predicates to quantifications and implications.
I.e. ImplicationOrder.instPartialOrder.rel P Q
becomes
∀ x y, P x y → Q x y
.
In the premise of the Park induction principle (lfp_le_of_le_monotone
) we use a monotone map defining the predicate in the eta expanded form. In such a case, besides desugaring the predicate, we need to perform a weak head reduction.
The optional parameter reduceConclusion
(false by default) indicates whether we need to perform this reduction.
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
Instances For
Returns true if name
defined by partial_fixpoint
, the first in its mutual group,
and all functions are defined using the CCPO
instance for Option
.
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.Elab.PartialFixpoint.isPartialCorrectnessName env name = (pure false).run
Instances For
Given motive : α → β → γ → Prop
, construct a proof of
admissible (fun f => ∀ x y r, f x y = r → motive x y r)
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.