]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/lib/lambda/subterms/booleanized.ma
decentralized notation in lambda
[helm.git] / matita / matita / lib / lambda / subterms / booleanized.ma
index d247ee73f41e19e1e050823c2fd3e1fafafe1dbd..cc6f1e9806db60c74fc3c9d394e0e708ff8f1799 100644 (file)
 
 include "lambda/subterms/boolean.ma".
 
+include "lambda/notation/functions/projectsame_2.ma".
+
+include "lambda/xoa/ex_4_3.ma".
+
 (* BOOLEANIZED SUBSET (EMPTY OR FULL) ***************************************)
 
 definition booleanized: bool → subterms → subterms ≝
@@ -22,10 +26,6 @@ definition booleanized: bool → subterms → subterms ≝
 interpretation "booleanized (subterms)"
    'ProjectSame b F = (booleanized b F).
 
-notation "hvbox( { term 46 b } ⇕ break term 46 F)"
-   non associative with precedence 46
-   for @{ 'ProjectSame $b $F }.
-
 lemma booleanized_inv_vref: ∀j,c,b,F. {b}⇕ F = {c}#j →
                             ∃∃b1. b = c & F = {b1}#j.
 #j #c #b #F #H