equal
deleted
inserted
replaced
1 (* ID: $Id$ *) |
1 (* ID: $Id$ *) |
2 theory Examples imports Main Binomial begin |
2 theory Examples imports Main Binomial begin |
3 |
3 |
4 ML "reset eta_contract" |
4 ML "Unsynchronized.reset eta_contract" |
5 ML "Pretty.setmargin 64" |
5 ML "Pretty.setmargin 64" |
6 |
6 |
7 text{*membership, intersection *} |
7 text{*membership, intersection *} |
8 text{*difference and empty set*} |
8 text{*difference and empty set*} |
9 text{*complement, union and universal set*} |
9 text{*complement, union and universal set*} |