src/HOL/Algebra/abstract/Abstract.thy
author huffman
Thu, 28 May 2009 13:43:45 -0700
changeset 31286 424874813840
parent 27541 9e585e99b494
child 35849 b5522b51cb1e
permissions -rw-r--r--
merged

(*
    Summary theory of the development of abstract algebra
    $Id$
    Author: Clemens Ballarin, started 17 July 1997
*)

theory Abstract
imports RingHomo Field
begin

end