X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Flibrary%2Falgebra%2Fgroups.ma;h=9ab695239665e8418d6279f8f1609334e7ddada1;hb=e1e31e9c6a0bcdc60ace7e2e650cb8d719d07e33;hp=ea345bc5469356224e3f102453264e0c3fa34542;hpb=37a7215f61ea70095a18f3e1135934343e66ad56;p=helm.git diff --git a/matita/library/algebra/groups.ma b/matita/library/algebra/groups.ma index ea345bc54..9ab695239 100644 --- a/matita/library/algebra/groups.ma +++ b/matita/library/algebra/groups.ma @@ -190,7 +190,7 @@ for @{ 'subgroupimage $H $x }. interpretation "Subgroup image" 'subgroupimage H x = (cic:/matita/algebra/groups/image.con _ _ - (cic:/matita/algebra/groups/morphism_of_subgroup.con _ H) x). + (cic:/matita/algebra/groups/morphism_OF_subgroup.con _ H) x). definition member_of_subgroup ≝ λG.λH:subgroup G.λx:G.∃y.x=y \sub H. @@ -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); @@ -316,10 +316,11 @@ record normal_subgroup (G:Group) : Type ≝ theorem foo: ∀G.∀H:normal_subgroup G.∀x.x*H=H*x. *) - +(* theorem member_of_left_coset_mk_left_coset_x_H_a_to_member_of_left_coset_mk_left_coset_y_H_b_to_member_of_left_coset_mk_left_coset_op_x_y_H_op_a_b: ∀G.∀H:normal_subgroup G.∀x,y,a,b. a ∈ (x*H) → b ∈ (y*H) → (a·b) ∈ ((x·y)*H). intros; simplify; -qed. \ No newline at end of file +qed. +*)