]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambda_delta/Basic_2/grammar/term_simple.ma
- notation fix for reducible and normal forms
[helm.git] / matita / matita / contribs / lambda_delta / Basic_2 / grammar / term_simple.ma
index 8f7c70374a92d17368d12cd7bd9242be881b2a15..557299afd7f4176ac394a29c3dc79e708395302b 100644 (file)
@@ -25,12 +25,12 @@ interpretation "simple (term)" 'Simple T = (simple T).
 
 (* Basic inversion lemmas ***************************************************)
 
-fact simple_inv_bind_aux: â\88\80T. ð\9d\95\8a[T] → ∀J,W,U. T = ⓑ{J} W. U → False.
+fact simple_inv_bind_aux: â\88\80T. ð\9d\90\92[T] → ∀J,W,U. T = ⓑ{J} W. U → False.
 #T * -T
 [ #I #J #W #U #H destruct
 | #I #V #T #J #W #U #H destruct
 ]
 qed.
 
-lemma simple_inv_bind: â\88\80I,V,T. ð\9d\95\8a[ⓑ{I} V. T] → False.
+lemma simple_inv_bind: â\88\80I,V,T. ð\9d\90\92[ⓑ{I} V. T] → False.
 /2 width=6/ qed-.