]> matita.cs.unibo.it Git - helm.git/commitdiff
fixed
authorEnrico Tassi <enrico.tassi@inria.fr>
Tue, 11 Jul 2006 08:06:53 +0000 (08:06 +0000)
committerEnrico Tassi <enrico.tassi@inria.fr>
Tue, 11 Jul 2006 08:06:53 +0000 (08:06 +0000)
matita/library/algebra/groups.ma

index 884e0c582e67d434c2f058ba83dd0a7fa7de54b0..9ab695239665e8418d6279f8f1609334e7ddada1 100644 (file)
@@ -296,7 +296,7 @@ qed.
 
 (*CSC: here the coercion Type_of_Group cannot be omitted. Why? *)
 theorem in_x_mk_left_coset_x_H:
- ∀G.∀x:Type_of_Group G.∀H:subgroup G.x ∈ (x*H).
+ ∀G.∀x:Type_OF_Group G.∀H:subgroup G.x ∈ (x*H).
 intros;
 simplify;
 apply (ex_intro ? ? 1);