mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-19 09:12:34 +03:00
23 lines
633 B
Plaintext
23 lines
633 B
Plaintext
1/1: Building RecordDoc (RecordDoc.idr)
|
|
RecordDoc>
|
|
RecordDoc> record RecordDoc.A : Type -> Type
|
|
Totality: total
|
|
Visibility: private
|
|
Constructor: __mkA : _
|
|
Projection: .anA : A a -> a
|
|
RecordDoc> record RecordDoc.Tuple : Type -> Type -> Type
|
|
Totality: total
|
|
Visibility: private
|
|
Constructor: __mkTuple : _
|
|
Projections:
|
|
.proj1 : Tuple a b -> a
|
|
.proj2 : Tuple a b -> b
|
|
RecordDoc> record RecordDoc.Singleton : a -> Type
|
|
Totality: total
|
|
Visibility: private
|
|
Constructor: __mkSingleton : _
|
|
Projections:
|
|
0 .equal : (rec : Singleton v) -> value rec = v
|
|
.value : Singleton v -> a
|
|
RecordDoc> Bye for now!
|