Equations
- One or more equations did not get rendered due to their size.
Instances For
Checks consistency of a clique of TerminationHints:
- If not all have a hint, the hints are ignored (log error)
- None have both
termination_by
andnontermination
(throw error) - If one has
structural
orpartialFixpoint
, check that all have it (else throw error) - A
structural
should not have adecreasing_by
(else log error)
Equations
- One or more equations did not get rendered due to their size.
Instances For
Elaborates the TerminationHint
in the clique to TerminationMeasures
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.Elab.shouldUsepartialFixpoint preDefs = preDefs.any fun (preDef : Lean.Elab.PreDefinition) => preDef.termination.partialFixpoint?.isSome
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.