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
- One or more equations did not get rendered due to their size.
Instances For
Equations
Instances For
A docComment
parses a "documentation comment" like /-- foo -/
. This is not treated like
a regular comment (that is, as whitespace); it is parsed and forms part of the syntax tree structure.
At parse time, docComment
checks the value of the doc.verso
option. If it is true, the contents
are parsed as Verso markup. If not, the contents are treated as plain text or Markdown. Use
plainDocComment
to always treat the contents as plain text.
A plain text doc comment node contains a /--
atom and then the remainder of the comment, foo -/
in this example. Use TSyntax.getDocString
to extract the body text from a doc string syntax node.
A Verso comment node contains the /--
atom, the document's syntax tree, and a closing -/
atom.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A docComment
parses a "documentation comment" like /-- foo -/
. This is not treated like
a regular comment (that is, as whitespace); it is parsed and forms part of the syntax tree structure.
At parse time, docComment
checks the value of the doc.verso
option. If it is true, the contents
are parsed as Verso markup. If not, the contents are treated as plain text or Markdown. Use
plainDocComment
to always treat the contents as plain text.
A plain text doc comment node contains a /--
atom and then the remainder of the comment, foo -/
in this example. Use TSyntax.getDocString
to extract the body text from a doc string syntax node.
A Verso comment node contains the /--
atom, the document's syntax tree, and a closing -/
atom.
Equations
Instances For
Equations
Instances For
Equations
Instances For
Built-in parsers #
by tac
constructs a term of the expected type by running the tactic(s) tac
.
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
Instances For
Instances For
Equations
Instances For
Instances For
Instances For
A type universe. Type ≡ Type 0
, Type u ≡ Sort (u + 1)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A specific universe in Lean's infinite hierarchy of universes.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The sorry
term is a temporary placeholder for a missing proof or value.
The syntax is intended for stubbing-out incomplete parts of a value or proof while still having a syntactically correct skeleton.
Lean will give a warning whenever a declaration uses sorry
, so you aren't likely to miss it,
but you can double check if a declaration depends on sorry
by looking for sorryAx
in the output
of the #print axioms my_thm
command, the axiom used by the implementation of sorry
.
"Go to definition" on sorry
in the Infoview will go to the source position where it was introduced, if such information is available.
Each sorry
is guaranteed to be unique, so for example the following fails:
example : (sorry : Nat) = sorry := rfl -- fails
See also the sorry
tactic, which is short for exact sorry
.
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
A placeholder for an implicit lambda abstraction's variable. The lambda abstraction is scoped to the surrounding parentheses.
For example, (· + ·)
is equivalent to fun x y => x + y
. Tuple notation and type ascription notation also serve as scopes.
Note that (· : ty)
expands to ((fun x => x) : ty)
, so ty
should be a function type.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Type ascription notation: (0 : Int)
instructs Lean to process 0
as a value of type Int
.
An empty type ascription (e :)
elaborates e
without the expected type.
This is occasionally useful when Lean's heuristics for filling arguments from the expected type
do not yield the right result.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Parentheses, used for grouping expressions (e.g., a * (b + c)
).
Can also be used for creating simple functions when combined with ·
. Here are some examples:
(· + 1)
is shorthand forfun x => x + 1
(· + ·)
is shorthand forfun x y => x + y
(f · a b)
is shorthand forfun x => f x a b
(h (· + 1) ·)
is shorthand forfun x => h (fun y => y + 1) x
- also applies to other parentheses-like notations such as
(·, 1)
and(· : Nat → Nat)
Equations
- One or more equations did not get rendered due to their size.
Instances For
The anonymous constructor ⟨e, ...⟩
is equivalent to c e ...
if the
expected type is an inductive type with a single constructor c
.
If more terms are given than c
has parameters, the remaining arguments
are turned into a new anonymous constructor application. For example,
⟨a, b, c⟩ : α × (β × γ)
is equivalent to ⟨a, ⟨b, c⟩⟩
.
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
Instances For
A sufficesDecl
represents everything that comes after the suffices
keyword:
an optional x :
, then a term ty
, then from val
or by tac
.
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
- One or more equations did not get rendered due to their size.
Instances For
@x
disables automatic insertion of implicit parameters of the constant x
.
@e
for any term e
also disables the insertion of implicit lambdas at this position.
Equations
- One or more equations did not get rendered due to their size.
Instances For
.(e)
marks an "inaccessible pattern", which does not influence evaluation of the pattern match, but may be necessary for type-checking.
In contrast to regular patterns, e
may be an arbitrary term of the appropriate type.
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
- 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
Useful for syntax quotations. Note that generic patterns such as `(matchAltExpr| | ... => $rhs)
should also
work with other rhsParser
s (of arity 1).
Instances For
Equations
- Lean.Parser.Term.instCoeTSyntaxConsSyntaxNodeKindMkStr4Nil_lean = { coe := fun (stx : Lean.TSyntax `Lean.Parser.Term.matchAltExpr) => { raw := stx.raw } }
Equations
- One or more equations did not get rendered due to their size.
Instances For
matchDiscr
matches a "match discriminant", either h : tm
or tm
, used in match
as
match h1 : e1, e2, h3 : e3 with ...
.
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
- 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
- One or more equations did not get rendered due to their size.
Instances For
Pattern matching. match e, ... with | p, ... => f | ...
matches each given
term e
against each pattern p
of a match alternative. When all patterns
of an alternative match, the match
term evaluates to the value of the
corresponding right-hand side f
with the pattern variables bound to the
respective matched values.
If used as match h : e, ... with | p, ... => f | ...
, h : e = p
is available
within f
.
When not constructing a proof, match
does not automatically substitute variables
matched on in dependent variables' types. Use match (generalizing := true) ...
to
enforce this.
Syntax quotations can also be used in a pattern match.
This matches a Syntax
value against quotations, pattern variables, or _
.
Quoted identifiers only match identical identifiers - custom matching such as by the preresolved names only should be done explicitly.
Syntax.atom
s are ignored during matching by default except when part of a built-in literal.
For users introducing new atoms, we recommend wrapping them in dedicated syntax kinds if they
should participate in matching.
For example, in
syntax "c" ("foo" <|> "bar") ...
foo
and bar
are indistinguishable during matching, but in
syntax foo := "foo"
syntax "c" (foo <|> "bar") ...
they are not.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Empty match/ex falso. nomatch e
is of arbitrary type α : Sort u
if
Lean can show that an empty set of patterns is exhaustive given e
's type,
e.g. because it has no constructors.
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
Structure instance. { x := e, ... }
assigns e
to field x
, which may be
inherited. If e
is itself a variable called x
, it can be elided:
fun y => { x := 1, y }
.
A structure update of an existing value can be given via with
:
{ point with x := 1 }
.
The structure type can be specified if not inferable:
{ x := 1, y := 2 : Point }
.
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
- 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
- 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
- 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
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
- One or more equations did not get rendered due to their size.
Instances For
Indicates that an argument to a function marked @[extern]
is borrowed.
Being borrowed only affects the ABI and runtime behavior of the function when compiled or interpreted. From the perspective of Lean's type system, this annotation has no effect. It similarly has no effect on functions not marked @[extern]
.
When a function argument is borrowed, the function does not consume the value. This means that the function will not decrement the value's reference count or deallocate it, and the caller is responsible for doing so.
Please see https://lean-lang.org/doc/reference/latest/find/?domain=Verso.Genre.Manual.section&name=ffi-borrowing for a complete description.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A literal of type Name
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A resolved name literal. Evaluates to the full name of the given constant if existent in the current context, or else fails.
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
- One or more equations did not get rendered due to their size.
Instances For
Equations
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.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
letDecl
matches the body of a let declaration let f x1 x2 := e
,
let pat := e
(where pat
is an arbitrary term) or let f | pat1 => e1 | pat2 => e2 ...
(a pattern matching declaration), except for the let
keyword itself.
let rec
declarations are not handled here.
Equations
- One or more equations did not get rendered due to their size.
Instances For
+postponeValue
causes the body of the let
to be elaborated before the value.
Equations
- One or more equations did not get rendered due to their size.
Instances For
+usedOnly
causes unused let
s bindings to be eliminated.
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
- 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
let (eq := h) x := v; ...
adds the equality h : x = v
to the context while elaborating the body.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Instances For
Configuration options for let
tactics.
Equations
- One or more equations did not get rendered due to their size.
Instances For
let
is used to declare a local definition. Example:
let x := 1
let y := x + 1
x + y
Since functions are first class citizens in Lean, you can use let
to declare
local functions too.
let double := fun x => 2*x
double (double 3)
For recursive definitions, you should use let rec
.
You can also perform pattern matching using let
. For example,
assume p
has type Nat × Nat
, then you can write
let (x, y) := p
x + y
The anaphoric let let := v
defines a variable called this
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
let_delayed x := v; b
is similar to let x := v; b
, but b
is elaborated before v
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
let
-declaration that is only included in the elaborated term if variable is still there.
It is often used when building macros.
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
- One or more equations did not get rendered due to their size.
Instances For
attrKind
matches ("scoped" <|> "local")?
, used before an attribute like @[local simp]
.
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
- One or more equations did not get rendered due to their size.
Instances For
Specify a termination measure for recursive functions.
termination_by a - b
indicates that termination of the currently defined recursive function follows
because the difference between the arguments a
and b
decreases.
If the function takes further argument after the colon, you can name them as follows:
def example (a : Nat) : Nat → Nat → Nat :=
termination_by b c => a - b
By default, a termination_by
clause will cause the function to be constructed using well-founded
recursion. The syntax termination_by structural a
(or termination_by structural _ c => c
)
indicates the function is expected to be structural recursive on the argument. In this case
the body of the termination_by
clause must be one of the function's parameters.
If omitted, a termination measure will be inferred. If written as termination_by?
,
the inferred termination measure will be suggested.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Specify a termination measure for recursive functions.
termination_by a - b
indicates that termination of the currently defined recursive function follows
because the difference between the arguments a
and b
decreases.
If the function takes further argument after the colon, you can name them as follows:
def example (a : Nat) : Nat → Nat → Nat :=
termination_by b c => a - b
By default, a termination_by
clause will cause the function to be constructed using well-founded
recursion. The syntax termination_by structural a
(or termination_by structural _ c => c
)
indicates the function is expected to be structural recursive on the argument. In this case
the body of the termination_by
clause must be one of the function's parameters.
If omitted, a termination measure will be inferred. If written as termination_by?
,
the inferred termination measure will be suggested.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Defines a possibly non-terminating function as a fixed-point in a suitable partial order.
Such a function is compiled as if it was marked partial
, but its equations are provided as
theorems, so that it can be verified.
In general it accepts functions whose return type has a Lean.Order.CCPO
instance and whose
definition is Lean.Order.monotone
with regard to its recursive calls.
Common special cases are
- Functions whose type is inhabited a-priori (as with
partial
), and where all recursive calls are in tail-call position. - Monadic in certain “monotone chain-complete monads” (in particular,
Option
) composed using the bind operator and other supported monadic combinators.
By default, the monotonicity proof is performed by the compositional monotonicity
tactic. Using
the syntax partial_fixpoint monotonicity by $tac
the proof can be done manually.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Defines a coinductive predicate using lattice theory, based on the Knaster-Tarski fixpoint theorem.
This feature constructs coinductive predicates by leveraging the lattice structure on Prop
and ensures correctness through monotonicity.
The coinductive predicate is defined as the greatest fixed point of a monotone function on Prop
.
By default, monotonicity is verified automatically. However, users can provide custom proofs of monotonicity if needed.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Defines an inductive predicate using lattice theory, based on the Knaster-Tarski fixpoint theorem.
This feature constructs inductive predicates by leveraging the lattice structure on Prop
and ensures correctness through monotonicity.
The inductive predicate is defined as the least fixed point of a monotone function on Prop
.
By default, monotonicity is verified automatically. However, users can provide custom proofs of monotonicity if needed.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Manually prove that the termination measure (as specified with termination_by
or inferred)
decreases at each recursive call.
By default, the tactic decreasing_tactic
is used.
Forces the use of well-founded recursion and is hence incompatible with
termination_by structural
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Termination hints are termination_by
and decreasing_by
, in that order.
Equations
- One or more equations did not get rendered due to their size.
Instances For
letRecDecl
matches the body of a let-rec declaration: a doc comment, attributes, and then
a let declaration without the let
keyword, such as /-- foo -/ @[simp] bar := 1
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
letRecDecls
matches letRecDecl,+
, a comma-separated list of let-rec declarations (see letRecDecl
).
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
A named subsection of where ... finally
. In the future, sections such as decreasing_by
might become
syntactic sugar for an where ... finally
subsection | decreasing => ...
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The finally
section trailing a where
opens a tactic block to fill in ?hole
s in the definition body.
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
- 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
unsafe t : α
is an expression constructor which allows using unsafe declarations inside the
body of t : α
, by creating an auxiliary definition containing t
and using implementedBy
to
wrap it in a safe interface. It is required that α
is nonempty for this to be sound,
but even beyond that, an unsafe
block should be carefully inspected for memory safety because
the compiler is unable to guarantee the safety of the operation.
For example, the evalExpr
function is unsafe, because the compiler cannot guarantee that when
you call evalExpr Foo ``Foo e
that the type Foo
corresponds to the name Foo
, but in a
particular use case, we can ensure this, so unsafe (evalExpr Foo ``Foo e)
is a correct usage.
Equations
- One or more equations did not get rendered due to their size.
Instances For
binrel% r a b
elaborates r a b
as a binary relation using the type propagation protocol in Lean.Elab.Extra
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
binrel_no_prop% r a b
is similar to binrel% r a b
, but it coerces Prop
arguments into Bool
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
binop% f a b
elaborates f a b
as a binary operation using the type propagation protocol in Lean.Elab.Extra
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
binop_lazy%
is similar to binop% f a b
, but it wraps b
as a function from Unit
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
leftact% f a b
elaborates f a b
as a left action using the type propagation protocol in Lean.Elab.Extra
.
In particular, it is like a unary operation with a fixed parameter a
, where only the right argument b
participates in the operator coercion elaborator.
Equations
- One or more equations did not get rendered due to their size.
Instances For
rightact% f a b
elaborates f a b
as a right action using the type propagation protocol in Lean.Elab.Extra
.
In particular, it is like a unary operation with a fixed parameter b
, where only the left argument a
participates in the operator coercion elaborator.
Equations
- One or more equations did not get rendered due to their size.
Instances For
unop% f a
elaborates f a
as a unary operation using the type propagation protocol in Lean.Elab.Extra
.
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
- One or more equations did not get rendered due to their size.
Instances For
A macro which evaluates to the name of the currently elaborating declaration.
Equations
- One or more equations did not get rendered due to their size.
Instances For
private_decl% e
elaborates e
in a private context and wraps the result in a helper def
.
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
- 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
- One or more equations did not get rendered due to their size.
Instances For
value_of% x
elaborates to the value of x
, which can be a local or global definition.
Equations
- One or more equations did not get rendered due to their size.
Instances For
clear% x; e
elaborates x
after clearing the free variable x
from the local context.
If x
cannot be cleared (due to dependencies), it will keep x
without failing.
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
- 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
- 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
Helper parser for marking match
-alternatives that should not trigger errors if unused.
We use them to implement macro_rules
and elab_rules
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
In a function application, ..
notation inserts zero or more _
placeholders.
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
The extended field notation e.f
is roughly short for T.f e
where T
is the type of e
.
More precisely,
- if
e
is of a function type,e.f
is translated toFunction.f (p := e)
wherep
is the first explicit parameter of function type - if
e
is of a named typeT ...
and there is a declarationT.f
(possibly fromexport
),e.f
is translated toT.f (p := e)
wherep
is the first explicit parameter of typeT ...
- otherwise, if
e
is of a structure type, the above is repeated for every base type of the structure.
The field index notation e.i
, where i
is a positive number,
is short for accessing the i
-th field (1-indexed) of e
if it is of a structure type.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Parser.Term.completion = Lean.Parser.trailingNode `Lean.Parser.Term.completion 1024 0 (Lean.Parser.checkNoWsBefore >> Lean.Parser.symbol ".")
Instances For
Equations
- Lean.Parser.Term.arrow = Lean.Parser.trailingNode `Lean.Parser.Term.arrow 1024 0 (Lean.Parser.checkPrec 25 >> Lean.Parser.unicodeSymbol " → " " -> " >> Lean.Parser.termParser 25)
Instances For
Syntax kind for syntax nodes representing the field of a projection in the InfoTree
.
Specifically, the InfoTree
node for a projection s.f
contains a child InfoTree
node
with syntax (Syntax.node .none identProjKind #[`f])
.
This is necessary because projection syntax cannot always be detected purely syntactically
(s.f
may refer to either the identifier s.f
or a projection s.f
depending on
the available context).
Equations
- Lean.Parser.Term.identProjKind = `Lean.Parser.Term.identProj
Instances For
Equations
- Lean.Parser.Term.isIdent stx = (stx.isAntiquot || stx.isIdent)
Instances For
x.{u, ...}
explicitly specifies the universes u, ...
of the constant x
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
x@e
or x@h:e
matches the pattern e
and binds its value to the identifier x
.
If present, the identifier h
is bound to a proof of x = e
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
e |>.x
is a shorthand for (e).x
.
It is especially useful for avoiding parentheses with repeated applications.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Parser.Term.pipeCompletion = Lean.Parser.trailingNode `Lean.Parser.Term.pipeCompletion Lean.Parser.minPrec 0 (Lean.Parser.symbol " |>.")
Instances For
h ▸ e
is a macro built on top of Eq.rec
and Eq.symm
definitions.
Given h : a = b
and e : p a
, the term h ▸ e
has type p b
.
You can also view h ▸ e
as a "type casting" operation
where you change the type of e
by using h
.
The macro tries both orientations of h
. If the context provides an
expected type, it rewrites the expected type, else it rewrites the type of e`.
See the Chapter "Quantifiers and Equality" in the manual "Theorem Proving in Lean" for additional information.
Equations
- Lean.Parser.Term.subst = Lean.Parser.trailingNode `Lean.Parser.Term.subst 75 0 (Lean.Parser.symbol " ▸ " >> Lean.Parser.sepBy1 (Lean.Parser.termParser 75) " ▸ ")
Instances For
Instances For
Equations
- Lean.Parser.Term.instCoeTSyntaxConsSyntaxNodeKindMkStr4Nil_lean_1 = { coe := fun (s : Lean.TSyntax `Lean.Parser.Term.bracketedBinderF) => { raw := s.raw } }
panic! msg
formally evaluates to @Inhabited.default α
if the expected type
α
implements Inhabited
.
At runtime, msg
and the file position are printed to stderr unless the C
function lean_set_panic_messages(false)
has been executed before. If the C
function lean_set_exit_on_panic(true)
has been executed before, the process is
then aborted.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A shorthand for panic! "unreachable code has been reached"
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
dbg_trace e; body
evaluates to body
and prints e
(which can be an
interpolated string literal) to stderr. It should only be used for debugging.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Instances For
A state monad that uses an actual mutable reference cell (i.e. an ST.Ref
).
This is syntax, rather than a function, to make it easier to use. Its elaborator synthesizes an
appropriate parameter for the underlying monad's ST
effects, then passes it to StateRefT'
.
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
- One or more equations did not get rendered due to their size.
Instances For
Implementation of the show_term
term elaborator.
Equations
- One or more equations did not get rendered due to their size.
Instances For
match_expr
support.
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
- 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
- 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
Throws an error exception, tagging the associated message as a named error with the specified name
and validating that an associated error explanation exists. The message may be passed as an
interpolated string or a MessageData
term. The result of getRef
is used as position information.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Throws an error exception, tagging the associated message as a named error with the specified name
and validating that an associated error explanation exists. The error name must be followed by a
Syntax
at which the error is to be thrown. The message is the final argument and may be passed as
an interpolated string or a MessageData
term.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Logs an error, tagging the message as a named error with the specified name and validating that an
associated error explanation exists. The message may be passed as an interpolated string or a
MessageData
term. The result of getRef
is used as position information.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Logs an error, tagging the message as a named error with the specified name and validating that an
associated error explanation exists. The error name must be followed by a Syntax
at which the
error is to be logged. The message is the final argument and may be passed as an interpolated string
or a MessageData
term.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Logs a warning, tagging the message as a named diagnostic with the specified name and validating
that an associated error explanation exists. The message may be passed as an interpolated string or
a MessageData
term. The result of getRef
is used as position information.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Logs a warning, tagging the message as a named diagnostic with the specified name and validating
that an associated error explanation exists. The error name must be followed by a Syntax
at which
the warning is to be logged. The message is the final argument and may be passed as an interpolated
string or a MessageData
term.
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
- One or more equations did not get rendered due to their size.