src/HOL/Algebra/Bij.thy
changeset 16417 9bc16273c2d4
parent 14963 d584e32f7d46
child 20318 0e0ea63fe768
     1.1 --- a/src/HOL/Algebra/Bij.thy	Fri Jun 17 11:35:35 2005 +0200
     1.2 +++ b/src/HOL/Algebra/Bij.thy	Fri Jun 17 16:12:49 2005 +0200
     1.3 @@ -5,7 +5,7 @@
     1.4  
     1.5  header {* Bijections of a Set, Permutation Groups, Automorphism Groups *}
     1.6  
     1.7 -theory Bij = Group:
     1.8 +theory Bij imports Group begin
     1.9  
    1.10  constdefs
    1.11    Bij :: "'a set \<Rightarrow> ('a \<Rightarrow> 'a) set"