src/HOL/Algebra/AbelCoset.thy
changeset 26203 9625f3579b48
parent 23463 9953ff53cc64
child 26310 f8a7fac36e13
--- a/src/HOL/Algebra/AbelCoset.thy	Wed Mar 05 21:33:59 2008 +0100
+++ b/src/HOL/Algebra/AbelCoset.thy	Wed Mar 05 21:42:21 2008 +0100
@@ -185,7 +185,7 @@
 
 lemma (in additive_subgroup) is_additive_subgroup:
   shows "additive_subgroup H G"
-by fact
+by (rule additive_subgroup_axioms)
 
 lemma additive_subgroupI:
   includes struct G
@@ -225,7 +225,7 @@
 
 lemma (in abelian_subgroup) is_abelian_subgroup:
   shows "abelian_subgroup H G"
-by fact
+by (rule abelian_subgroup_axioms)
 
 lemma abelian_subgroupI:
   assumes a_normal: "normal H \<lparr>carrier = carrier G, mult = add G, one = zero G\<rparr>"