src/HOL/Algebra/abstract/Abstract.thy
author wenzelm
Fri, 13 Mar 2009 19:53:09 +0100
changeset 30509 e19d5b459a61
parent 27541 9e585e99b494
child 35849 b5522b51cb1e
permissions -rw-r--r--
more regular method setup via SIMPLE_METHOD;

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

theory Abstract
imports RingHomo Field
begin

end