]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambda_delta/Basic_2/grammar/term_simple.ma
component "reducibility" updated to new syntax!
[helm.git] / matita / matita / contribs / lambda_delta / Basic_2 / grammar / term_simple.ma
index be508e49cddbe70d9f22c3ce04b74f8d2b32f8eb..be4811eebd0819ee1de128e67779a5b076b7205d 100644 (file)
@@ -16,7 +16,7 @@ include "Basic_2/grammar/term.ma".
 
 (* SIMPLE (NEUTRAL) TERMS ***************************************************)
 
-inductive simple: term → Prop ≝
+inductive simple: predicate term ≝
    | simple_atom: ∀I. simple (𝕒{I})
    | simple_flat: ∀I,V,T. simple (𝕗{I} V. T)
 .
@@ -33,4 +33,4 @@ fact simple_inv_bind_aux: ∀T. 𝕊[T] → ∀J,W,U. T = 𝕓{J} W. U → False
 qed.
 
 lemma simple_inv_bind: ∀I,V,T. 𝕊[𝕓{I} V. T] → False.
-/2 width=6/ qed.
+/2 width=6/ qed-.