File tree Expand file tree Collapse file tree 4 files changed +20
-30
lines changed Expand file tree Collapse file tree 4 files changed +20
-30
lines changed Original file line number Diff line number Diff line change 1
- Theorem thm4 : 1 = 1. Proof . reflexivity. Qed .
1
+ Theorem thm4 : 1 = 1. Proof . Admitted .
Original file line number Diff line number Diff line change 1
- Require Import Solution.
2
-
3
- Theorem thm1 : 1 = 1 + 0. Proof . admit. Admitted .
4
- Print Assumptions thm1.
5
-
6
- Parameter thm2 : 1 + 0 = 0 + 1.
7
- Print Assumptions thm2.
8
-
9
- Theorem thm3 : 1 = 0 + 1. Proof . rewrite <- thm2. exact thm1. Qed .
10
- Print Assumptions thm3.
11
-
12
- Theorem thm4_check : 1 = 1.
13
- Proof .
14
- exact thm4.
15
- Print Assumptions thm4.
16
- Qed .
1
+ Require Solution.
2
+ From CW Require Import Loader.
3
+
4
+ CWGroup "Solution.thm4".
5
+ CWTest "should have the correct type".
6
+ CWAssert Solution.thm4 : (1 = 1).
7
+ CWTest "should be closed under the global context".
8
+ CWAssert Solution.thm4 Assumes.
9
+ CWEndGroup.
Original file line number Diff line number Diff line change 1
- Theorem plus_n_O : forall n:nat, n = n + 0.
2
- Proof .
3
- intros n.
4
- induction n.
5
- - reflexivity.
6
- - simpl. rewrite <- IHn. reflexivity.
7
- Qed .
1
+ Theorem thm4 : 1 = 1. Proof . reflexivity. Qed .
Original file line number Diff line number Diff line change 1
- Require Import Solution.
2
- Theorem plus_n_O_check : forall n:nat, n = n + 0.
3
- Proof .
4
- exact plus_n_O.
5
- Print Assumptions plus_n_O.
6
- Qed .
1
+ Require Solution.
2
+ From CW Require Import Loader.
3
+
4
+ CWGroup "Solution.thm4".
5
+ CWTest "should have the correct type".
6
+ CWAssert Solution.thm4 : (1 = 1).
7
+ CWTest "should be closed under the global context".
8
+ CWAssert Solution.thm4 Assumes.
9
+ CWEndGroup.
You can’t perform that action at this time.
0 commit comments