src/HOL/Algebra/abstract/PID.thy
author haftmann
Mon, 20 Jul 2009 08:32:07 +0200
changeset 32075 e8e0fb5da77a
parent 29665 2b956243d123
child 35849 b5522b51cb1e
permissions -rw-r--r--
merged

(*
    Principle ideal domains
    Author: Clemens Ballarin, started 5 October 1999
*)

theory PID imports Ideal2 begin

instance pid < factorial
  apply intro_classes
  apply (erule pid_irred_imp_prime)
  done

end