mirror of
https://github.com/idris-lang/Idris2.git
synced 2025-01-01 16:12:26 +03:00
[ 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:
parent
fce45c5762
commit
a39783be8e
@ -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
|
||||
|
@ -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`.
|
||||
|
@ -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
|
||||
|
Loading…
Reference in New Issue
Block a user