]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/library/algebra/groups.ma
maction support added to notation, adopted for = AKA = \sub t
[helm.git] / helm / software / matita / library / algebra / groups.ma
index 29324c4aa748f9d4cf4f8b6d215c6d23f59bb2e0..d6e77ae8d0fa6a36404b7d084911e12602c234de 100644 (file)
@@ -218,8 +218,8 @@ definition left_coset_eq ≝
  λG.λC,C':left_coset G.
   ∀x.((element ? C)·x \sub (subgrp ? C)) ∈ C'.
   
-interpretation "Left cosets equality" 'eq C C' =
- (cic:/matita/algebra/groups/left_coset_eq.con _ C C').
+interpretation "Left cosets equality" 'eq C C' =
+ (cic:/matita/algebra/groups/left_coset_eq.con t C C').
 
 definition left_coset_disjoint ≝
  λG.λC,C':left_coset G.
@@ -287,7 +287,7 @@ theorem in_x_mk_left_coset_x_H:
  ∀G.∀x:Type_OF_Group G.∀H:subgroup G.x ∈ (x*H).
 intros;
 simplify;
-apply (ex_intro ? ? 1);
+apply (ex_intro ? ? );
 rewrite > morphism_to_eq_f_1_1;
 rewrite > (e_is_right_unit ? G);
 reflexivity.