aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/typeclasses/clrewrite.v
diff options
context:
space:
mode:
authorGravatar glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-09-17 15:58:14 +0000
committerGravatar glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-09-17 15:58:14 +0000
commit61ccbc81a2f3b4662ed4a2bad9d07d2003dda3a2 (patch)
tree961cc88c714aa91a0276ea9fbf8bc53b2b9d5c28 /test-suite/typeclasses/clrewrite.v
parent6d3fbdf36c6a47b49c2a4b16f498972c93c07574 (diff)
Delete trailing whitespaces in all *.{v,ml*} files
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12337 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/typeclasses/clrewrite.v')
-rw-r--r--test-suite/typeclasses/clrewrite.v20
1 files changed, 10 insertions, 10 deletions
diff --git a/test-suite/typeclasses/clrewrite.v b/test-suite/typeclasses/clrewrite.v
index 2978fda26..f21acd4cb 100644
--- a/test-suite/typeclasses/clrewrite.v
+++ b/test-suite/typeclasses/clrewrite.v
@@ -15,7 +15,7 @@ Section Equiv.
Qed.
Tactic Notation "simpl" "*" := auto || relation_tac.
-
+
Goal eqA x y -> eqA y x /\ True.
intros H ; clrewrite H.
split ; simpl*.
@@ -27,13 +27,13 @@ Section Equiv.
Qed.
Goal eqA x y -> eqA y z -> eqA x y.
- intros H.
+ intros H.
clrewrite H.
intro. refl.
Qed.
-
+
Goal eqA x y -> eqA z y -> eqA x y.
- intros H.
+ intros H.
clrewrite <- H at 2.
clrewrite <- H at 1.
intro. refl.
@@ -54,7 +54,7 @@ Section Equiv.
clrewrite <- H.
refl.
Qed.
-
+
Goal eqA x y -> True /\ True /\ False /\ eqA x x -> True /\ True /\ False /\ eqA x y.
Proof.
intros.
@@ -70,12 +70,12 @@ Section Trans.
Variables x y z w : A.
Tactic Notation "simpl" "*" := auto || relation_tac.
-
+
(* Typeclasses eauto := debug. *)
Goal R x y -> R y x -> R y y -> R x x.
Proof with auto.
- intros H H' H''.
+ intros H H' H''.
clrewrite <- H' at 2.
clrewrite H at 1...
@@ -86,11 +86,11 @@ Section Trans.
clrewrite H.
refl.
Qed.
-
+
Goal R x y -> R z y -> R x y.
- intros H.
+ intros H.
clrewrite <- H at 2.
- intro.
+ intro.
clrewrite H at 1.
Abort.