From: Claudio Sacerdoti Coen Date: Tue, 7 Mar 2006 18:21:39 +0000 (+0000) Subject: This simplify seems to diverge! X-Git-Tag: 0.4.95@7852~1617 X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=commitdiff_plain;h=37a7215f61ea70095a18f3e1135934343e66ad56;hp=c0044e3f39e3af51abe8971cfdfdb71e2b9cd7bb;p=helm.git This simplify seems to diverge! --- diff --git a/matita/library/algebra/groups.ma b/matita/library/algebra/groups.ma index 360e75c9f..ea345bc54 100644 --- a/matita/library/algebra/groups.ma +++ b/matita/library/algebra/groups.ma @@ -294,6 +294,7 @@ rewrite > (e_is_right_unit ? H); reflexivity. 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). intros; @@ -302,4 +303,23 @@ apply (ex_intro ? ? 1); rewrite > morphism_to_eq_f_1_1; rewrite > (e_is_right_unit ? G); reflexivity. +qed. + +(* Normal Subgroups *) + +record normal_subgroup (G:Group) : Type ≝ + { ns_subgroup:> subgroup G; + normal:> ∀x:G.∀y:ns_subgroup.(x·y \sub ns_subgroup·x \sup -1) ∈ ns_subgroup + }. + +(*CSC: I have not defined yet right cosets +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