]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/lib/formal_topology/o-algebra.ma
support for nat-labeled reflexive and transitive closure added to lambdadelta
[helm.git] / matita / matita / lib / formal_topology / o-algebra.ma
index 496485975f0db459fc03f0e05dd225dd8fc7dd45..70473755095490011616866e83c78f411fc36a22 100644 (file)
@@ -13,7 +13,7 @@
 (**************************************************************************)
 
 include "formal_topology/categories.ma".
-
+(*
 inductive bool : Type[0] := true : bool | false : bool.
 
 lemma BOOL : objs1 SET.
@@ -440,3 +440,4 @@ qed.
 lemma oa_overlap_sym': ∀o:OA.∀U,V:o. (U >< V) = (V >< U).
  intros; split; intro; apply oa_overlap_sym; assumption.
 qed.
+*)