]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/lib/re/re.ma
update in lib
[helm.git] / matita / matita / lib / re / re.ma
index af0e921a6b9a1be5cbabe311860e2fb8d7d09c8b..8ba714b82592f01047735b685663a64ed200f3d5 100644 (file)
@@ -13,6 +13,7 @@
 (**************************************************************************)
 
 include "re/lang.ma".
+include "basics/core_notation/card_1.ma".
 
 (* The type re of regular expressions over an alphabet $S$ is the smallest 
 collection of objects generated by the following constructors: *)
@@ -128,8 +129,7 @@ let rec forget (S: DeqSet) (l : pitem S) on l: re S ≝
   | po E1 E2 ⇒ (forget ? E1) + (forget ? E2)
   | pk E ⇒ (forget ? E)^* ].
  
-(* notation < "|term 19 e|" non associative with precedence 70 for @{'forget $e}.*)
-interpretation "forget" 'norm a = (forget ? a).
+interpretation "forget" 'card a = (forget ? a).
 
 lemma erase_dot : ∀S.∀e1,e2:pitem S. |e1 · e2| = c ? (|e1|) (|e2|).
 // qed.