]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/nlibrary/logic/equality.ma
Implementation of ndestruct tactic (including destruction of constructor forms
[helm.git] / helm / software / matita / nlibrary / logic / equality.ma
index 715423143e7185debaf41b69046ba5e1ccde202b..b92f92f66c6fd60be592bfab75360be0a2458d0f 100644 (file)
@@ -28,6 +28,11 @@ nlemma eq_rect_CProp0_r:
  #A; #a; #P; #p; #x0; #p0; napply (eq_rect_CProp0_r' ??? p0); nassumption.
 nqed.
 
+nlemma eq_ind_r :
+ ∀A.∀a.∀P: ∀x:A. eq ? x a → Prop. P a (refl A a) → ∀x.∀p:eq ? x a.P x p.
+ #A; #a; #P; #p; #x0; #p0; napply (eq_rect_CProp0_r' ??? p0); nassumption.
+nqed.
+
 interpretation "leibnitz's equality" 'eq t x y = (eq t x y).
 
 interpretation "leibnitz's non-equality" 'neq t x y = (Not (eq t x y)).