From 711b00a770c30056019a2b7204903e7fb5981940 Mon Sep 17 00:00:00 2001 From: Claudio Sacerdoti Coen Date: Sun, 1 Feb 2009 20:46:43 +0000 Subject: [PATCH] Towards fullness. --- .../overlap/r-o-basic_pairs.ma | 30 ++++++++++++++++++- 1 file changed, 29 insertions(+), 1 deletion(-) diff --git a/helm/software/matita/contribs/formal_topology/overlap/r-o-basic_pairs.ma b/helm/software/matita/contribs/formal_topology/overlap/r-o-basic_pairs.ma index f90b8bbba..729f2894b 100644 --- a/helm/software/matita/contribs/formal_topology/overlap/r-o-basic_pairs.ma +++ b/helm/software/matita/contribs/formal_topology/overlap/r-o-basic_pairs.ma @@ -23,7 +23,35 @@ lemma rOR_full : ∀s,t:rOBP.∀f:arrows2 OBTop (OR (ℱ_2 s)) (OR (ℱ_2 t)). exT22 ? (λg:arrows2 rOBP s t. map_arrows2 ?? OR ?? (ℳ_2 g) = f). -intros; cases f (h H1 H2); clear f; simplify; +intro; cases s (s_2 s_1 s_eq); clear s; cases s_eq; clear s_eq s_2; +intro; cases t (t_2 t_1 t_eq); clear t; cases t_eq; clear t_eq t_2; +whd in ⊢ (%→?); whd in ⊢ (? (? ? ? ? %) (? ? ? ? %)→?); +intro; whd in s_1 t_1; +letin y ≝ (f⎻* ); clearbody y; + change in y with (carr2 (POW (form s_1) ⇒ POW (form t_1))); +alias symbol "Vdash" = "basic pair relation for subsets (non applied)". +letin z ≝ (image ?? (⊩ \sub s_1)); clearbody z; +change in z with ((POW (concr s_1) → POW (form s_1))); + (*change in z with (carr2 (POW (concr s_1) ⇒ POW (form s_1)));*) + + letin R ≝ (y ∘ z); + + letin R ≝ (f* );∘ (⊩ \sub s_1)); + + +whd in ⊢ (? % ?→?); +whd in ⊢ (? % ?→?); cases s_eq; intro; whd in f; +simplify; +intro; cases f (g H1 H2); clear f; exists; + [ constructor 1; + [ + | unfold F1; simplify; + | + ] + | + ] + + cases f (h H1 H2); clear f; simplify; change in ⊢ (? ? (λg:?.? ? ? (? ? ? %) ?)) with (o_continuous_relation_of_o_relation_pair ?? (ℳ_2 g)). -- 2.39.2