[ fix #2721 ] Don't reflow doc lines

I don't think there's a good solution at least until we start
parsing these comments so let's just keep them as they were written
by the library writer.
This commit is contained in:
Guillaume Allais 2022-10-18 16:17:07 +01:00 committed by G. Allais
parent fce45c5762
commit a39783be8e
3 changed files with 4 additions and 4 deletions

View File

@ -262,7 +262,7 @@ getDocsForName fc n config
showDoc : Config -> (Name, String) -> Core (Doc IdrisDocAnn)
reflowDoc : String -> List (Doc IdrisDocAnn)
reflowDoc str = map (indent 2 . reflow) (lines str)
reflowDoc str = map (indent 2 . pretty0) (lines str)
showTotal : Totality -> Maybe (Doc IdrisDocAnn)
showTotal tot

View File

@ -81,8 +81,8 @@ Main> interface Prelude.Show : Type -> Type
A value should produce parentheses around itself if and only if the given
precedence context is greater than or equal to the precedence of the
outermost operation represented in the produced `String`. *This is
different from Haskell*, which requires it to be strictly greater. `Open`
outermost operation represented in the produced `String`. *This is
different from Haskell*, which requires it to be strictly greater. `Open`
should thus always produce *no* outermost parens, `App` should always
produce outermost parens except on atomic values and those that provide
their own bracketing, like `Pair` and `List`.

View File

@ -8,7 +8,7 @@ Data.String.singleton : Char -> String
Prelude.Show.show : Char -> String
Prelude.Cast.cast : Char -> String
Main> Prelude.const : a -> b -> a
Constant function. Ignores its second argument.
Constant function. Ignores its second argument.
Totality: total
Visibility: public export
Main> Builtin.fromChar : Char -> Char