- useDecide : Bool
Check whether any of the hypotheses is an empty type.
emptyType : BoolWhen checking for empty types,
searchFuel
specifies the number of goals visited.searchFuel : NatSupport for hypotheses such as
h : (x y : Nat) (ys : List Nat) → x = 0 → y::ys = [a, b, c] → False
This kind of hypotheses appear when proving conditional equation theorems for match expressions.genDiseq : Bool
@[inline]
Equations
- Lean.Meta.ElimEmptyInductive.instMonadBacktrackSavedStateM = { saveState := liftM Lean.Meta.saveState, restoreState := fun s => liftM (Lean.Meta.SavedState.restore s) }
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Meta.contradiction
(mvarId : Lean.MVarId)
(config : optParam Lean.Meta.Contradiction.Config { useDecide := true, emptyType := true, searchFuel := 16, genDiseq := false })
:
Equations
- One or more equations did not get rendered due to their size.