src/HOL/Algebra/ROOT.ML
author haftmann
Tue, 29 Jul 2008 14:20:22 +0200
changeset 27695 033732c90ebd
parent 24153 1a4607b7ad24
child 27713 95b36bfe7fc4
permissions -rw-r--r--
Haskell now living in the RealWorld

(*
    The Isabelle Algebraic Library
    $Id$
    Author: Clemens Ballarin, started 24 September 1999
*)

(* Preliminaries from set and number theory *)
no_document use_thys ["FuncSet", "Primes", "Binomial"];


(*** New development, based on explicit structures ***)

use_thys [
  (* Groups *)
  "FiniteProduct",      (* Product operator for commutative groups *)
  "Sylow",              (* Sylow's theorem *)
  "Bij",                (* Automorphism Groups *)

  (* Rings *)
  "UnivPoly",           (* Rings and polynomials *)
  "IntRing"             (* Ideals and residue classes *)
];


(*** Old development, based on axiomatic type classes.
     Will be withdrawn in future. ***)

no_document use_thys [
  "abstract/Abstract",  (*The ring theory*)
  "poly/Polynomial"     (*The full theory*)
];