Idris2/tests/idris2/misc/docs002/expected

27 lines
691 B
Plaintext
Raw Normal View History

1/1: Building Doc (Doc.idr)
Doc> MkSimpleRec : Int -> String -> SimpleRec
MkWrappedInt : Int -> WrappedInt
SimpleRec : Type
WrappedInt : Type
a : SimpleRec -> Int
b : SimpleRec -> String
hello : Int -> Int
world : Nat -> Nat
.a : SimpleRec -> Int
.b : SimpleRec -> String
Doc> Doc.NS.NestedNS.Foo : Type
A type of Foo
Visibility: private
2021-08-19 13:38:14 +03:00
Doc> data Doc.WrappedInt : Type
Totality: total
Visibility: public export
Constructor: MkWrappedInt : Int -> WrappedInt
2021-08-19 13:38:14 +03:00
Doc> record Doc.SimpleRec : Type
Totality: total
Visibility: public export
Constructor: MkSimpleRec : Int -> String -> SimpleRec
Projections:
.a : SimpleRec -> Int
.b : SimpleRec -> String
Doc> Bye for now!