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=cf07c50b03a49344eb4cbe2e1bc18fcef880b9e9;hp=789c7c9c50df894f8c4cb5270278f7009d6afa49;hpb=9791cd146bc0b8df953aee7bb8a3df60553b530c;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 789c7c9c5..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. @@ -47,4 +48,4 @@ lemma Or_symmetric: symmetric ? Or. unfold; intros (x y H); cases H; [right|left] assumption; qed. - \ No newline at end of file +