]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/dama/constructive_higher_order_relations.ma
matitadep sould be ok, outputs warning regarding issues and
[helm.git] / matita / dama / constructive_higher_order_relations.ma
index 789c7c9c50df894f8c4cb5270278f7009d6afa49..8d195396cc455efc20ec7c0875b7e4264d2e6d5e 100644 (file)
 (*                                                                        *)
 (**************************************************************************)
 
-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
+