]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambda_delta/ground_2/xoa_props.ma
- we introduced the pointer_step rc in the perspective of proving
[helm.git] / matita / matita / contribs / lambda_delta / ground_2 / xoa_props.ma
index 121eb7e741cdb2f4d37bd5d1b73dd80ed8166730..71216d1c4dee1cc0795580468c082e67dfb47473 100644 (file)
 (*                                                                        *)
 (**************************************************************************)
 
-include "Ground_2/xoa_notation.ma".
-include "Ground_2/xoa.ma".
+include "basics/logic.ma".
+include "ground_2/xoa_notation.ma".
+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/