]> matita.cs.unibo.it Git - helm.git/commitdiff
Experiment...
authorClaudio Sacerdoti Coen <claudio.sacerdoticoen@unibo.it>
Mon, 28 Sep 2009 09:59:15 +0000 (09:59 +0000)
committerClaudio Sacerdoti Coen <claudio.sacerdoticoen@unibo.it>
Mon, 28 Sep 2009 09:59:15 +0000 (09:59 +0000)
helm/software/matita/nlibrary/logic/cprop.ma

index e18811da416feab641aab7f79f6b2324fe5ee9b7..d857ba6a72942fabd1898feff2934a0b832c1e72 100644 (file)
@@ -52,7 +52,14 @@ ndefinition and_morphism: binary_morphism1 CPROP CPROP CPROP.
      | napply (H4 K2)]##]
 nqed.
 
-unification hint 0 ≔ A,B ⊢ fun21 … and_morphism A B ≡ And A B.
+(*unification hint 0 ≔ A,B ⊢ fun21 … and_morphism A B ≡ And A B.*)
+unification hint 0 ≔ A,B ⊢ fun21 … (mk_binary_morphism1 … And (prop21 … and_morphism)) A B ≡ And A B.
+
+(*nlemma test: ∀A,A',B: CProp[0]. A=A' → (B ∨ A) = B → (B ∧ A) ∧ B.
+ #A; #A'; #B; #H1; #H2;
+ napply (. ((#‡H1)‡H2^-1)); nnormalize;
+nqed.*)
+
 
 (*nlemma test: ∀A,A',B: CProp[0]. A=A' → (B ∨ A) = B → (B ∧ A) ∧ B.
  #A; #A'; #B; #H1; #H2;