changeset 2440 | 0a36825b16c1 |
parent 2436 | 3885dc2669f9 |
child 2454 | 9ffee4eb1ae1 |
2439:cc6e281d8f72 | 2440:0a36825b16c1 |
---|---|
1 theory TypeVarsTest |
1 theory TypeVarsTest |
2 imports "../NewParser" |
2 imports "../NewParser" |
3 begin |
3 begin |
4 |
4 |
5 atom_decl name |
5 atom_decl name |
6 declare [[STEPS = 21]] |
6 declare [[STEPS = 100]] |
7 |
7 |
8 class s1 |
8 class s1 |
9 class s2 |
9 class s2 |
10 |
10 |
11 nominal_datatype ('a, 'b) lam = |
11 nominal_datatype ('a, 'b) lam = |