File: test_stepwise.v

package info (click to toggle)
proofgeneral 4.5-3
  • links: PTS, VCS
  • area: main
  • in suites: sid, trixie
  • size: 5,172 kB
  • sloc: lisp: 33,783; makefile: 388; sh: 118; perl: 109
file content (38 lines) | stat: -rw-r--r-- 651 bytes parent folder | download
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
Definition trois := 3. (*test-definition*)
Print trois.
Eval compute in 10 * trois * trois.
 


Lemma easy_proof : forall A : Prop, A -> A.
Proof using .
  intros A.
  intros proof_of_A. (*test-insert*)
  exact proof_of_A.
Qed. (*test-lemma*)

Section failSection.
  Local Unset Ltac Backtrace.
  Goal False.
  Proof. (*FailNoTrace*)
    Fail (now auto).
    auto.
  Abort.

  Local Set Ltac Backtrace.
  Goal False. (*FailTrace*) 
    Fail (now auto).
    auto.
  Abort.
End failSection.


Lemma false_proof : forall A B : bool, A = B. 
Proof.
  intros A B.
  destruct A.
  destruct B.
  reflexivity. (*error*)
  reflexivity.
Qed. (*test-lemma2*)