author | wenzelm |
Mon, 01 Mar 2010 17:12:43 +0100 | |
changeset 35414 | cc8e4276d093 |
parent 29665 | 2b956243d123 |
child 35849 | b5522b51cb1e |
permissions | -rw-r--r-- |
7998 | 1 |
(* |
2 |
Principle ideal domains |
|
3 |
Author: Clemens Ballarin, started 5 October 1999 |
|
4 |
*) |
|
5 |
||
20318
0e0ea63fe768
Restructured algebra library, added ideals and quotient rings.
ballarin
parents:
17479
diff
changeset
|
6 |
theory PID imports Ideal2 begin |
7998 | 7 |
|
17479 | 8 |
instance pid < factorial |
9 |
apply intro_classes |
|
10 |
apply (erule pid_irred_imp_prime) |
|
11 |
done |
|
7998 | 12 |
|
13 |
end |