]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/lib/formal_topology/o-algebra.ma
backport of WIP on \lambda\delta to matita 0.99.3
[helm.git] / matita / matita / lib / formal_topology / o-algebra.ma
index 496485975f0db459fc03f0e05dd225dd8fc7dd45..61a784605dfbaec75c5254a6e6fa1463bcc466c0 100644 (file)
@@ -12,8 +12,9 @@
 (*                                                                        *)
 (**************************************************************************)
 
+include "basics/core_notation/comprehension_2.ma".
 include "formal_topology/categories.ma".
-
+(*
 inductive bool : Type[0] := true : bool | false : bool.
 
 lemma BOOL : objs1 SET.
@@ -440,3 +441,4 @@ qed.
 lemma oa_overlap_sym': ∀o:OA.∀U,V:o. (U >< V) = (V >< U).
  intros; split; intro; apply oa_overlap_sym; assumption.
 qed.
+*)