X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=helm%2Fsoftware%2Fmatita%2Fdama%2Fconstructive_higher_order_relations.ma;h=8d195396cc455efc20ec7c0875b7e4264d2e6d5e;hb=7abdf2f1764ba67a48f0829f7a9813ce7426b0c6;hp=cf58e2640ec6a6472dd9731286cd9d0bfcdb9b9b;hpb=475120bb8ccfe5877bbe294006170ed7ab0b1fcd;p=helm.git diff --git a/helm/software/matita/dama/constructive_higher_order_relations.ma b/helm/software/matita/dama/constructive_higher_order_relations.ma index cf58e2640..8d195396c 100644 --- a/helm/software/matita/dama/constructive_higher_order_relations.ma +++ b/helm/software/matita/dama/constructive_higher_order_relations.ma @@ -12,9 +12,10 @@ (* *) (**************************************************************************) -set "baseuri" "cic:/matita/constructive_higher_order_relations". + include "constructive_connectives.ma". +include "higher_order_defs/relations.ma". definition cotransitive ≝ λC:Type.λlt:C→C→Type.∀x,y,z:C. lt x y → lt x z ∨ lt z y. @@ -35,3 +36,16 @@ definition associative ≝ definition commutative ≝ λC:Type.λop:C→C→C.λeq:C→C→Type.∀x,y. eq (op x y) (op y x). + +alias id "antisymmetric" = "cic:/matita/higher_order_defs/relations/antisymmetric.con". +theorem antisimmetric_to_cotransitive_to_transitive: + ∀C:Type.∀le:C→C→Prop. antisymmetric ? le → cotransitive ? le → transitive ? le. +intros (T f Af cT); unfold transitive; intros (x y z fxy fyz); +lapply (cT ??z fxy) as H; cases H; [assumption] cases (Af ? ? fyz H1); +qed. + +lemma Or_symmetric: symmetric ? Or. +unfold; intros (x y H); cases H; [right|left] assumption; +qed. + +