Skip to content
Snippets Groups Projects
Commit 25057899 authored by Adam's avatar Adam
Browse files

Remove tests mentioning core

parent 032e2739
Branches core-up
No related tags found
No related merge requests found
...@@ -15,7 +15,8 @@ Section base_logic_tests. ...@@ -15,7 +15,8 @@ Section base_logic_tests.
Context {M : ucmra}. Context {M : ucmra}.
Implicit Types P Q R : uPred M. Implicit Types P Q R : uPred M.
Lemma test_random_stuff (P1 P2 P3 : nat -> uPred M) : (*TODO*)
(*Lemma test_random_stuff (P1 P2 P3 : nat -> uPred M) :
|- forall (x y : nat) a b, |- forall (x y : nat) a b,
x ≡ y -> x ≡ y ->
<#> (uPred_ownM (a ⋅ b) -* <#> (uPred_ownM (a ⋅ b) -*
...@@ -38,7 +39,7 @@ Section base_logic_tests. ...@@ -38,7 +39,7 @@ Section base_logic_tests.
iApply ("H3" $! _ 0 with "[$]"). iApply ("H3" $! _ 0 with "[$]").
- iSplit; first done. iApply "H2". iLeft. iApply "H2". by iRight. - iSplit; first done. iApply "H2". iLeft. iApply "H2". by iRight.
- done. - done.
Qed. Qed.*)
Lemma test_iFrame_pure (x y z : M) : Lemma test_iFrame_pure (x y z : M) :
x -> y z |-@{uPredI M} x /\ x /\ y z. x -> y z |-@{uPredI M} x /\ x /\ y z.
......
...@@ -12,7 +12,8 @@ Section base_logic_tests. ...@@ -12,7 +12,8 @@ Section base_logic_tests.
Context {M : ucmra}. Context {M : ucmra}.
Implicit Types P Q R : uPred M. Implicit Types P Q R : uPred M.
Lemma test_random_stuff (P1 P2 P3 : nat uPred M) : (*TODO*)
(*Lemma test_random_stuff (P1 P2 P3 : nat → uPred M) :
⊢ ∀ (x y : nat) a b, ⊢ ∀ (x y : nat) a b,
x ≡ y → x ≡ y →
□ (uPred_ownM (a ⋅ b) -∗ □ (uPred_ownM (a ⋅ b) -∗
...@@ -35,7 +36,7 @@ Section base_logic_tests. ...@@ -35,7 +36,7 @@ Section base_logic_tests.
iApply ("H3" $! _ 0 with "[$]"). iApply ("H3" $! _ 0 with "[$]").
- iSplit; first done. iApply "H2". iLeft. iApply "H2". by iRight. - iSplit; first done. iApply "H2". iLeft. iApply "H2". by iRight.
- done. - done.
Qed. Qed.*)
Lemma test_iFrame_pure (x y z : M) : Lemma test_iFrame_pure (x y z : M) :
x y z -∗ ( x x y z : uPred M). x y z -∗ ( x x y z : uPred M).
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Please register or to comment