]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/dama/divisible_group.ma
snapshot
[helm.git] / helm / software / matita / dama / divisible_group.ma
index 4f54545c8fbd74c6817037fdba164b6580f9615f..3a79b11bbd969a884307f4a6a86d08e63cbcfff8 100644 (file)
@@ -50,8 +50,8 @@ qed.
 lemma div1: ∀G:dgroup.∀x:G.x/O ≈ x.
 intro G; cases G; unfold divide; intros; simplify;
 cases (f x O); simplify; simplify in H; intro; apply H;
-apply (ap_rewl ???? (plus_comm ???));
-apply (ap_rewl ???w (zero_neutral ??)); assumption;
+apply (Ap≪ ? (plus_comm ???));
+apply (Ap≪ w (zero_neutral ??)); assumption;
 qed.
 
 lemma apmul_ap: ∀G:dgroup.∀x,y:G.∀n.S n * x # S n * y → x # y.