You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
Copy file name to clipboardExpand all lines: Manual/Defs.lean
+5-5Lines changed: 5 additions & 5 deletions
Original file line number
Diff line number
Diff line change
@@ -489,7 +489,7 @@ The headers and bodies of definitions are elaborated together.
489
489
If the header is incompletely specified (e.g. a parameter's type or the codomain is missing), then the body may provide sufficient information for the elaborator to reconstruct the missing parts.
490
490
However, {tech}[instanceimplicit]parametersmustbespecifiedintheheaderoras {tech}[sectionvariables].
Abbreviations are identical to definitions with {keyword}`def`, except they are {tech}[reducible].
522
522
523
523
```grammar
@@ -545,7 +545,7 @@ Unlike {tech}[axioms], opaque declarations can only be used for types that are i
545
545
Also unlike axioms, the inhabitant of the type is used in compiled code.
546
546
The {attr}`implemented_by` attribute can be used to instruct the compiler to emit a call to some other function as the compilation of an opaque constant.
Copy file name to clipboardExpand all lines: Manual/RecursiveDefs.lean
+1-1Lines changed: 1 addition & 1 deletion
Original file line number
Diff line number
Diff line change
@@ -490,7 +490,7 @@ semireducible
490
490
```grammar
491
491
irreducible
492
492
```
493
-
These attributes can only be applied globally in the same file as the definition being modified, but they may be {keywordOf attrInst parser:=Lean.Parser.Term.attrKind}`local`ly applied anywhere.
493
+
These attributes can only be applied globally in the same file as the definition being modified, but they may be {keywordOf attrInst (parser := Lean.Parser.Term.attrKind)}`local`ly applied anywhere.
Copy file name to clipboardExpand all lines: Manual/Terms.lean
+1-1Lines changed: 1 addition & 1 deletion
Original file line number
Diff line number
Diff line change
@@ -357,7 +357,7 @@ fun $x:ident : term => $t
357
357
```
358
358
:::
359
359
360
-
Function definitions defined with keywords such as {keywordOf Lean.Parser.Command.declaration parser:=Lean.Parser.Command.definition}`def` desugar to {keywordOf Lean.Parser.Term.fun}`fun`.
360
+
Function definitions defined with keywords such as {keywordOf Lean.Parser.Command.declaration (parser := Lean.Parser.Command.definition)}`def` desugar to {keywordOf Lean.Parser.Term.fun}`fun`.
361
361
Inductive type declarations, on the other hand, introduce new values with function types (constructors and type constructors) that cannot themselves be implemented using just {keywordOf Lean.Parser.Term.fun}`fun`.
0 commit comments