src/HOL/Algebra/abstract/Field.thy
author paulson
Mon, 05 Mar 2001 15:25:11 +0100
changeset 11193 851c90b23a9e
parent 11093 62c2e0af1d30
child 17479 68a7acb5f22e
permissions -rw-r--r--
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp

(*
    Properties of abstract class field
    $Id$
    Author: Clemens Ballarin, started 15 November 1997
*)

Field = Factor + PID +

instance
  field < domain (field_one_not_zero, field_integral)

instance
  field < factorial (TrueI, field_fact_prime)

end