Please enable JavaScript in your browser!
首頁
探索
說明
登入
caryoscelus
/
agda
關註
1
讚好
0
複刻
0
Files
問題管理
0
合併請求
0
Wiki
目錄樹:
ce9b406819
分支列表
標籤列表
js_amd
js_amd_patch
working
agda
/
test
/
LaTeXAndHTML
/
succeed
/
Issue3020.agda
Issue3020.agda
115 B
文件歷史
原始文件
1
2
3
4
5
6
7
8
9
10
11
12
13
record R : Set₁ where
field
A : Set
B : Set
B = A
field
C : Set
D : Set
D = A → B → C