diff options
Diffstat (limited to 'coq/example.v')
| -rw-r--r-- | coq/example.v | 6 |
1 files changed, 5 insertions, 1 deletions
diff --git a/coq/example.v b/coq/example.v index 5d55a2ae..6f92e279 100644 --- a/coq/example.v +++ b/coq/example.v @@ -9,7 +9,7 @@ $Id$ *) -Section sect. +Module sect. Goal (A,B:Prop)(A /\ B) -> (B /\ A). Intros A B H. @@ -32,5 +32,9 @@ End mod. Module Type newmod. Definition type1:=Set. + +Goal (n:nat)n=n. +Auto. +Save toto. End newmod. |
