changeset 2299 | 09bbed4f21d6 |
parent 2296 | 45a69c9cc4cc |
child 2302 | c6db12ddb60c |
2298:aead2aad845c | 2299:09bbed4f21d6 |
---|---|
3 begin |
3 begin |
4 |
4 |
5 atom_decl name |
5 atom_decl name |
6 |
6 |
7 ML {* print_depth 50 *} |
7 ML {* print_depth 50 *} |
8 declare [[STEPS = 5]] |
8 declare [[STEPS = 8]] |
9 |
9 |
10 |
10 |
11 nominal_datatype trm = |
11 nominal_datatype trm = |
12 Var "name" |
12 Var "name" |
13 | App "trm" "trm" |
13 | App "trm" "trm" |