]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/lib/formal_topology/relations.ma
- untranslated sections of "formal_topology" commented to make it compile
[helm.git] / matita / matita / lib / formal_topology / relations.ma
index 2ad35655e51756a1ceceda01182f1c126b0100f2..2d5d85a6be9a1dc0cca55b46d702694b655712a8 100644 (file)
@@ -13,7 +13,7 @@
 (**************************************************************************)
 
 include "formal_topology/subsets.ma".
-
+(*
 record binary_relation (A,B: SET) : Type[1] ≝
  { satisfy:> binary_morphism1 A B CPROP }.
 
@@ -323,4 +323,5 @@ theorem extS_singleton:
  intros; unfold extS; unfold ext; unfold singleton; simplify;
  split; intros 2; simplify; simplify in f; 
  [ cases f; cases e; cases x1; change in f2 with (x =_1 w); apply (. #‡f2); assumption;
- | split; try apply I; exists [apply x] split; try assumption; change with (x = x); apply rule #;] qed.
\ No newline at end of file
+ | split; try apply I; exists [apply x] split; try assumption; change with (x = x); apply rule #;] qed.
+*)