]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/contribs/ng_assembly/num/quatern_lemmas.ma
Release 0.5.9.
[helm.git] / helm / software / matita / contribs / ng_assembly / num / quatern_lemmas.ma
index a3ff945590970b1a501fc101ff12c068605cb6e6..c2c8a33998be710b0b0d4379f06a0c9dc4b3bc11 100755 (executable)
@@ -16,7 +16,7 @@
 (*                          Progetto FreeScale                            *)
 (*                                                                        *)
 (*   Sviluppato da: Ing. Cosimo Oliboni, oliboni@cs.unibo.it              *)
-(*   Sviluppo: 2008-2010                                                  *)
+(*   Ultima modifica: 05/08/2009                                          *)
 (*                                                                        *)
 (* ********************************************************************** *)
 
@@ -27,7 +27,6 @@ include "num/bool_lemmas.ma".
 (* QUATERNARI *)
 (* ********** *)
 
-(*
 ndefinition quatern_destruct_aux ≝
 Πn1,n2:quatern.ΠP:Prop.n1 = n2 →
  match eq_qu n1 n2 with [ true ⇒ P → P | false ⇒ P ].
@@ -39,7 +38,6 @@ ndefinition quatern_destruct : quatern_destruct_aux.
  nnormalize;
  napply (λx.x).
 nqed.
-*)
 
 nlemma eq_to_eqqu : ∀n1,n2.n1 = n2 → eq_qu n1 n2 = true.
  #n1; #n2; #H;
@@ -63,7 +61,7 @@ nlemma eqqu_to_eq : ∀n1,n2.eq_qu n1 n2 = true → n1 = n2.
  ncases n2;
  nnormalize;
  ##[ ##1,6,11,16: #H; napply refl_eq
- ##| ##*: #H; ndestruct (*napply (bool_destruct … H)*)
+ ##| ##*: #H; napply (bool_destruct … H)
  ##]
 nqed.