Skip to content

Conversation

david-christiansen
Copy link
Collaborator

No description provided.

pimotte and others added 30 commits May 12, 2025 21:46
This PR adds highlights to v4.19 release notes and reorganizes entries
in the extended list.
This PR adds highlights section to v4.20 release notes.
I needed this to get `main` working, so I can start a branch for the
`grind` manual.
…ng` error message (leanprover#459)

Example issue:

```
✖ [469/477] Building Manual.BuildTools.Elan
error: reference-manual/Manual/BuildTools/Elan.lean:226:0: Mismatched 'elan --help' output output:
                                                                                    ^^^^^^^^^^^^^
```

`main` branch:

```
Manual/Meta/ExpectString.lean:    logErrorAt expected m!"Mismatched {what} output:\n{Diff.linesToString diff}"
…
Manual/Meta/ElanCheck.lean:    discard <| expectString "'elan --help' output" str elanOutput (useLine := useLine) (preEq := String.trimRight)
Manual/Meta/ExpectString.lean:def expectString (what : String) (expected : StrLit) (actual : String)
Manual/Meta/LakeCheck.lean:    discard <| expectString "'lake --help' output" str lakeOutput (useLine := useLine)
Manual/Meta/LakeToml.lean:        discard <| expectString "elaborated configuration" expectedStr v (useLine := (·.any (!·.isWhitespace)))
```

This branch:

```
Manual/Meta/ExpectString.lean:    logErrorAt expected m!"Mismatched {what}:\n{Diff.linesToString diff}"
…
Manual/Meta/ElanCheck.lean:    discard <| expectString "'elan --help' output" str elanOutput (useLine := useLine) (preEq := String.trimRight)
Manual/Meta/ExpectString.lean:def expectString (what : String) (expected : StrLit) (actual : String)
Manual/Meta/LakeCheck.lean:    discard <| expectString "'lake --help' output" str lakeOutput (useLine := useLine)
Manual/Meta/LakeToml.lean:        discard <| expectString "elaborated configuration output" expectedStr v (useLine := (·.any (!·.isWhitespace)))
```

Co-authored-by: u <u@h>
The name of the `add` definition suggests that it can be used to
calculate the sum of two natural numbers, but in the current form, it is
always evaluated to the parameter `n` instead of `n+m`
…er#448)

Verso now ships KaTeX itself, so no need to include it here.
This reverts commit 423d015.

The manual is getting developed on nightly-testing, so that's the version that should be shown for the preview.
Lean PR 7428 brings a huge speedup to `simp` so we should be sure to
mention it!
@david-christiansen david-christiansen added the HTML available HTML has been generated for this PR label Jun 20, 2025
Copy link
Contributor

Preview for this PR is ready! 🎉 (also as a proofreading version). built with commit bcf63b0.

@david-christiansen david-christiansen merged commit 860abdb into leanprover:nightly-testing Jun 20, 2025
9 checks passed
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment
Labels
HTML available HTML has been generated for this PR
Projects
None yet
Development

Successfully merging this pull request may close these issues.

10 participants