aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib7
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-29 18:56:22 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-29 18:56:22 +0000
commit7ee14e9fb95e4e182f9983278275a6052d9b60da (patch)
tree9c0ad69b5eecc327f9344051e2fc737125c63ddd /contrib7
parentf4d66182ea20873db9bb15bc4ce0a6ec2738c323 (diff)
Deplacement des fichiers ancienne syntaxe dans theories7, contrib7 et states7
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5033 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib7')
-rw-r--r--contrib7/cc/.cvsignore1
-rw-r--r--contrib7/cc/CCSolve.v20
2 files changed, 21 insertions, 0 deletions
diff --git a/contrib7/cc/.cvsignore b/contrib7/cc/.cvsignore
new file mode 100644
index 000000000..c446fcb87
--- /dev/null
+++ b/contrib7/cc/.cvsignore
@@ -0,0 +1 @@
+*.v8
diff --git a/contrib7/cc/CCSolve.v b/contrib7/cc/CCSolve.v
new file mode 100644
index 000000000..30622aeaa
--- /dev/null
+++ b/contrib7/cc/CCSolve.v
@@ -0,0 +1,20 @@
+(***********************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * INRIA-Rocquencourt & LRI-CNRS-Orsay *)
+(* \VV/ *************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(***********************************************************************)
+
+(* $Id$ *)
+
+Tactic Definition CCsolve :=
+ Repeat (Match Context With
+ [ H: ?1 |- ?2] ->
+ Let Heq = FreshId "Heq" In
+ (Assert Heq:(?2==?1);[Congruence|(Rewrite Heq;Exact H)])
+ |[ H: ?1; G: ?2 -> ?3 |- ?] ->
+ Let Heq = FreshId "Heq" In
+ (Assert Heq:(?2==?1) ;[Congruence|
+ (Rewrite Heq in G;Generalize (G H);Clear G;Intro G)])).
+