]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/ground_2/xoa_props.ma
xoa: change in naming convenctions for existential quantifies
[helm.git] / matita / matita / contribs / lambdadelta / ground_2 / xoa_props.ma
index 71216d1c4dee1cc0795580468c082e67dfb47473..06bfbc739b7f091f55555fd45c6bff315ff7f42a 100644 (file)
@@ -19,7 +19,3 @@ include "ground_2/xoa.ma".
 interpretation "logical false" 'false = False.
 
 interpretation "logical true" 'true = True.
-
-lemma ex2_1_comm: ∀A0. ∀P0,P1:A0→Prop. (∃∃x0. P0 x0 & P1 x0) → ∃∃x0. P1 x0 & P0 x0.
-#A0 #P0 #P1 * /2 width=3/
-qed.