]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambda/preamble.ma
lstar removed from list.ma and placed in its own file
[helm.git] / matita / matita / contribs / lambda / preamble.ma
index 8e4b8fc962c0859991ec63c5c9c41e71d3e28ff9..c272595a2831f306ed7c12961cda21e2fa35bbf6 100644 (file)
@@ -28,10 +28,6 @@ notation "⊥"
   non associative with precedence 90
   for @{'false}.
 
-lemma ex2_1_commute: ∀A0. ∀P0,P1:A0→Prop. (∃∃x0. P0 x0 & P1 x0) → ∃∃x0. P1 x0 & P0 x0.
-#A0 #P0 #P1 * /2 width=3/
-qed.
-
 (* relations *)
 
 definition confluent1: ∀A. relation A → predicate A ≝ λA,R,a0.
@@ -42,6 +38,11 @@ definition confluent1: ∀A. relation A → predicate A ≝ λA,R,a0.
 definition confluent: ∀A. predicate (relation A) ≝ λA,R.
                       ∀a0. confluent1 … R a0.
 
+(* booleans *)
+
+definition is_false: predicate bool ≝ λb.
+                     false = b.
+
 (* arithmetics *)
 
 lemma lt_refl_false: ∀n. n < n → ⊥.