]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/matita/tests/unfold.ma
1. ProofEngineHelpers.locate_in_term, ProofEngineHelpers.locate_in_conjecture
[helm.git] / helm / matita / tests / unfold.ma
index ff68d5fd1e8cbb111bb13fda979665d60b49809e..c91ff18636999638c233c9844a8481c1b3a6f776 100644 (file)
@@ -21,9 +21,10 @@ lemma lem: \forall n. S (n + n) = (S n) + n.
  intro; reflexivity.
 qed.
 
-theorem trivial: \forall n. S (myplus n n) = (S n) + n.
- unfold myplus.
+theorem trivial: \forall n. S (myplus n n) = myplus (S n) n.
+ unfold myplus in \vdash \forall _.(? ? ? %).
  intro.
+ unfold myplus.
  rewrite > lem.
  reflexivity.
 qed.
\ No newline at end of file