src/HOL/Algebra/abstract/Abstract.thy
author blanchet
Wed, 28 Apr 2010 18:11:11 +0200
changeset 36550 f8da913b6c3a
parent 35849 b5522b51cb1e
permissions -rw-r--r--
make sure short theorem names are preferred to composite ones in Sledgehammer; this code used to work at some point

(*  Author: Clemens Ballarin, started 17 July 1997

Summary theory of the development of abstract algebra.
*)

theory Abstract
imports RingHomo Field
begin

end