- coe : α → β
- coe : α → β
Instances
- coe : α → β
- coe : α → β
- coe : β
Instances
- coe : α → β
Instances
Equations
- coeNotation = Lean.ParserDescr.node `coeNotation 1024 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol "↑") (Lean.ParserDescr.cat `term 1024))
instance
coeOfHeafOfTCOfTail
{α : Sort u}
{β : Sort v}
{δ : Sort w}
{γ : Sort w'}
[inst : CoeHead α β]
[inst : CoeTail δ γ]
[inst : CoeTC β δ]
:
CoeHTCT α γ
Equations
- coeOfHeafOfTCOfTail = { coe := fun a => CoeTail.coe (CoeTC.coe (CoeHead.coe a)) }
instance
coeOfHeadOfTC
{α : Sort u}
{β : Sort v}
{δ : Sort w}
[inst : CoeHead α β]
[inst : CoeTC β δ]
:
CoeHTCT α δ
Equations
- coeOfHeadOfTC = { coe := fun a => CoeTC.coe (CoeHead.coe a) }
instance
coeOfTCOfTail
{α : Sort u}
{β : Sort v}
{δ : Sort w}
[inst : CoeTail β δ]
[inst : CoeTC α β]
:
CoeHTCT α δ
Equations
- coeOfTCOfTail = { coe := fun a => CoeTail.coe (CoeTC.coe a) }
Equations
- coeSortToCoeTail = { coe := CoeSort.coe }
@[inline]
Equations
- boolToProp = { coe := fun b => b = true }
Equations
- decPropToBool p = { coe := decide p }
Equations
- subtypeCoe = { coe := fun v => v.val }
@[inline]
def
Lean.Internal.liftCoeM
{m : Type u → Type v}
{n : Type u → Type w}
{α : Type u}
{β : Type u}
[inst : MonadLiftT m n]
[inst : (a : α) → CoeT α a β]
[inst : Monad n]
(x : m α)
:
n β
Equations
- Lean.Internal.liftCoeM x = do let a ← liftM x pure a
@[inline]
def
Lean.Internal.coeM
{m : Type u → Type v}
{α : Type u}
{β : Type u}
[inst : (a : α) → CoeT α a β]
[inst : Monad m]
(x : m α)
:
m β
Equations
- Lean.Internal.coeM x = do let a ← x pure a
instance
instCoeDep
{α : Sort u_1}
{β : α → Sort u_2}
[inst : CoeFun α β]
(a : α)
:
CoeDep α a (β a)
Equations
- instCoeDep a = { coe := a }
Equations
- instCoeTail = { coe := fun a => a }
Equations
- instCoeTail_1 = { coe := fun a => a }