src/HOL/Algebra/abstract/Abstract.thy
author blanchet
Wed, 05 Sep 2012 11:08:18 +0200
changeset 49147 0da8120bd2aa
parent 35849 b5522b51cb1e
permissions -rw-r--r--
don't get confused by extraneous premisses

(*  Author: Clemens Ballarin, started 17 July 1997

Summary theory of the development of abstract algebra.
*)

theory Abstract
imports RingHomo Field
begin

end