changeset 58881 | b9556a055632 |
parent 55945 | e96383acecf9 |
child 60500 | 903bb1495239 |
58880:0baae4311a9f | 58881:b9556a055632 |
---|---|
1 (* Title: HOL/Library/Quotient_Syntax.thy |
1 (* Title: HOL/Library/Quotient_Syntax.thy |
2 Author: Cezary Kaliszyk and Christian Urban |
2 Author: Cezary Kaliszyk and Christian Urban |
3 *) |
3 *) |
4 |
4 |
5 header {* Pretty syntax for Quotient operations *} |
5 section {* Pretty syntax for Quotient operations *} |
6 |
6 |
7 theory Quotient_Syntax |
7 theory Quotient_Syntax |
8 imports Main |
8 imports Main |
9 begin |
9 begin |
10 |
10 |