]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/lib/tutorial/chapter7.ma
- pts_dummy/pts_dummy_new: non compiling parts commented out
[helm.git] / matita / matita / lib / tutorial / chapter7.ma
index 739afb52df7acd0ad2af9e964f98ce0fc4568daf..20b670018cc21de67fb8227e53ebe4cca692984e 100644 (file)
@@ -120,7 +120,10 @@ let rec forget (S: DeqSet) (l : pitem S) on l: re S ≝
   | pc E1 E2 ⇒ (forget ? E1) · (forget ? E2)
   | po E1 E2 ⇒ (forget ? E1) + (forget ? E2)
   | pk E ⇒ (forget ? E)^* ].
+
+(* Already in the library
+notation "| term 19 C |" with precedence 70 for @{ 'card $C }.
+*)
 interpretation "forget" 'card a = (forget ? a).
 
 lemma erase_dot : ∀S.∀e1,e2:pitem S. |e1 · e2| = c ? (|e1|) (|e2|).
@@ -304,4 +307,4 @@ lemma minus_eps_pre: ∀S.∀e:pre S. \sem{\fst e} =1 \sem{e}-{[ ]}.
     [/3/ | * * // #H1 #H2 @False_ind @(absurd …H1 H2)]
   |>sem_pre_false normalize in ⊢ (??%?); #w % [ /3/ | * // ]
   ]
-qed.
\ No newline at end of file
+qed.