@[class]
Instances of this typeclass
Instances of other typeclasses for has_orelse
- has_orelse.has_sizeof_inst
@[class]
- to_applicative : applicative f
- to_has_orelse : has_orelse f
- failure : Π {α : Type ?}, f α
Instances of this typeclass
- option.alternative
- tactic.alternative
- tactic.unsafe.type_context.type_context_alternative
- lean.parser.alternative
- state_t.alternative
- reader_t.alternative
- option_t.alternative
- conv.alternative
- smt_tactic.alternative
- list.alternative
- monad_io_is_alternative
- io_core_is_alternative
- old_conv.alternative
- set.alternative
- tactic.ring.ring_m.alternative
- tactic.ring_exp.ring_exp_m.alternative
- filter.alternative
- tactic.norm_fin.eval_fin_m.alternative
- parser.alternative
- computation.alternative
- finset.alternative
Instances of other typeclasses for alternative
- alternative.has_sizeof_inst
Equations
If the condition p
is decided to be false, then fail, otherwise, return unit.
Equations
- guard p = ite p (has_pure.pure unit.star()) failure