src/HOL/Algebra/abstract/Abstract.thy
author huffman
Sun, 28 Feb 2010 20:56:28 -0800
changeset 35481 7bb9157507a9
parent 27541 9e585e99b494
child 35849 b5522b51cb1e
permissions -rw-r--r--
add_domain_constructors takes iso_info record as argument

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

theory Abstract
imports RingHomo Field
begin

end