]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/lib/lambda/subterms/carrier.ma
decentralized notation in lambda
[helm.git] / matita / matita / lib / lambda / subterms / carrier.ma
index a15e11180958d5333974bdd4c13483513dbade25..3f4c0499181fa17b33cc40284fb184772c443677 100644 (file)
 include "lambda/terms/relocating_substitution.ma".
 include "lambda/subterms/relocating_substitution.ma".
 
+include "lambda/notation/functions/projectdown_1.ma".
+
+include "lambda/xoa/ex_2_2.ma".
+
 (* CARRIER (UNDERLYING TERM) ************************************************)
 
 let rec carrier F on F ≝ match F with
@@ -26,10 +30,6 @@ let rec carrier F on F ≝ match F with
 interpretation "carrier (subterms)"
    'ProjectDown F = (carrier F).
 
-notation "hvbox(⇓ term 46 F)"
-   non associative with precedence 46
-   for @{ 'ProjectDown $F }.
-
 lemma carrier_inv_vref: ∀j,F. ⇓F = #j → ∃b. F = {b}#j.
 #j * normalize
 [ #b #i #H destruct /2 width=2/