Commit
This commit does not belong to any branch on this repository, and may belong to a fork outside of the repository.
fix: redundant line breaks in trace messages (#571)
This PR ensures that there are no redundant line breaks when the trace formatter is including a newline at the end of a trace line. Example (from `whnfProj.lean`): ```lean import Lean def h (x : Nat) := x def f (x : Nat) := x + 1 def g (x : Nat) := (x, x+1).fst open Lean open Lean.Meta def tst (declName : Name) : MetaM Unit := do let c ← getConstInfo declName lambdaTelescope c.value! fun _ b => do trace[Meta.debug] "1. {b}" trace[Meta.debug] "2. {← withReducible <| whnf b}" trace[Meta.debug] "3. {← withReducibleAndInstances <| whnf b}" trace[Meta.debug] "4. {← withDefault <| whnf b}" pure () set_option trace.Meta.debug true #eval tst `f #eval tst `g ```
- Loading branch information