mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-19 01:01:59 +03:00
27 lines
691 B
Plaintext
27 lines
691 B
Plaintext
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
|
|
Doc> data Doc.WrappedInt : Type
|
|
Totality: total
|
|
Visibility: public export
|
|
Constructor: MkWrappedInt : Int -> WrappedInt
|
|
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!
|