changeset 58882 | 6e2010ab8bd9 |
parent 58614 | 7338eb25226c |
child 61797 | 458b4e3720ab |
58881:b9556a055632 | 58882:6e2010ab8bd9 |
---|---|
1 (* Title: HOL/Isar_Examples/Group_Context.thy |
1 (* Title: HOL/Isar_Examples/Group_Context.thy |
2 Author: Makarius |
2 Author: Makarius |
3 *) |
3 *) |
4 |
4 |
5 header \<open>Some algebraic identities derived from group axioms -- theory context version\<close> |
5 section \<open>Some algebraic identities derived from group axioms -- theory context version\<close> |
6 |
6 |
7 theory Group_Context |
7 theory Group_Context |
8 imports Main |
8 imports Main |
9 begin |
9 begin |
10 |
10 |