]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/lib/formal_topology/saturations.ma
- untranslated sections of "formal_topology" commented to make it compile
[helm.git] / matita / matita / lib / formal_topology / saturations.ma
index 02030e7cde3f2a2789a88f7f936e7bfc3ff98732..fab775bbeb91468866439cea34bdf5d4aa4c7c80 100644 (file)
@@ -13,7 +13,7 @@
 (**************************************************************************)
 
 include "formal_topology/relations.ma".
-
+(*
 definition is_saturation: ∀C:REL. Ω^C ⇒_1 Ω^C → CProp[1] ≝
  λC:REL.λA:Ω^C ⇒_1 Ω^C. ∀U,V. (U ⊆ A V) =_1 (A U ⊆ A V).
 
@@ -36,3 +36,4 @@ theorem saturation_idempotent: ∀C,A. is_saturation C A → ∀U. A (A U) = A U
   [ apply (if ?? (i ??)); apply subseteq_refl
   | apply saturation_expansive; assumption]
 qed.
+*)