fixed whitespace for *.md and .rst files

This commit is contained in:
stefan-hoeck 2021-01-22 14:30:42 +01:00 committed by G. Allais
parent 8b96614454
commit 29a6aa45e0
18 changed files with 44 additions and 54 deletions

View File

@ -85,5 +85,3 @@ Rather than using ``State`` and ``Exception`` directly, however,
we typically use interfaces to constrain the operations which are allowed
in a list of errors. Internally, ``State`` is implemented via an
``IORef``, primarily for performance reasons.

View File

@ -53,4 +53,3 @@ interfaces.
exceptionsstate
interfaces
linear

View File

@ -144,5 +144,3 @@ with any errors thrown by ``readFile``:
readMain fname = handle (readFile fname)
(\str => putStrLn $ "Success:\n" ++ show str)
(\err : IOError => putStrLn $ "Error: " ++ show err)

View File

@ -105,4 +105,3 @@ is ``NoThrow`` or ``MayThrow``. But, in practice, all applications
given to ``run`` will not throw at the top level, because the only
exception type available is the empty type ``Void``. Any exceptions
will have been introduced and handled inside the ``App``.

View File

@ -130,6 +130,3 @@ Also included in the prelude:
||| @ y the right side
(~=~) : (x : a) -> (y : b) -> Type
(~=~) x y = (x = y)

View File

@ -261,4 +261,3 @@ by using ``idris2 -client``.
More sophisticated support can be added by using the IDE protocol (yet to
be documented for Idris 2, but which mostly extends to protocol documented for
`Idris 1 <https://docs.idris-lang.org/en/latest/reference/ide-protocol.html>`_.