]> matita.cs.unibo.it Git - helm.git/commitdiff
fixed eliminator name
authorEnrico Tassi <enrico.tassi@inria.fr>
Wed, 2 Sep 2009 11:12:10 +0000 (11:12 +0000)
committerEnrico Tassi <enrico.tassi@inria.fr>
Wed, 2 Sep 2009 11:12:10 +0000 (11:12 +0000)
helm/software/matita/contribs/ng_assembly/common/theory.ma

index 70b12fcc5d17f4e456c2bfa0d7ddb2d8aea36aea..093c85e130b850525520cf97a6787be54b988415 100644 (file)
@@ -503,7 +503,7 @@ nlemma symmetric_eq: ∀A:Type. symmetric A (eq A).
  napply refl_eq.
 nqed.
 
-nlemma eq_elim_r: ∀A:Type.∀x:A.∀P:A → Prop.P x → ∀y:A.y=x → P y.
+nlemma eq_ind_r: ∀A:Type.∀x:A.∀P:A → Prop.P x → ∀y:A.y=x → P y.
  #A; #x; #P; #H; #y; #H1;
  nrewrite < (symmetric_eq … H1);
  napply H.