diff options
| author | Pierre Courtieu | 2003-02-03 14:36:13 +0000 |
|---|---|---|
| committer | Pierre Courtieu | 2003-02-03 14:36:13 +0000 |
| commit | 38bd477c79a5c7eb7d91df0575a6b469bde31d63 (patch) | |
| tree | 58ed94f15212c2125c7f9f8cf14e00fd32fc13ad /coq/example.v | |
| parent | 45e3d2559c4d57a41fe8784dc1a74467b6c6f50a (diff) | |
code cleaning + deals better with the new module system of Coq. Did
not test the fsfemacs. Will do before release.
Diffstat (limited to 'coq/example.v')
| -rw-r--r-- | coq/example.v | 21 |
1 files changed, 13 insertions, 8 deletions
diff --git a/coq/example.v b/coq/example.v index 6f92e279..5d076280 100644 --- a/coq/example.v +++ b/coq/example.v @@ -9,7 +9,7 @@ $Id$ *) -Module sect. +Section sect. Goal (A,B:Prop)(A /\ B) -> (B /\ A). Intros A B H. @@ -26,15 +26,20 @@ Recursive Tactic Definition bar := Idtac. Save and_comms. End sect. -Module mod. +Section newmod. Definition type1:=Set. -End mod. -Module Type newmod. -Definition type1:=Set. - -Goal (n:nat)n=n. -Auto. +Axiom A:False. +Goal (n:nat)(S n)=n. +Apply False_ind. +Exact A. Save toto. End newmod. +Extract Constant + +Lemma Lem : (S O)=O. +AutoRewrite [db]. + +Hint Rewrite [toto] in db. +AutoRewrite [db]. |
