Skip to content

Commit

Permalink
Some clean up
Browse files Browse the repository at this point in the history
  • Loading branch information
lyonel2017 committed Dec 18, 2024
1 parent 3281ee9 commit 99ff0ce
Show file tree
Hide file tree
Showing 2 changed files with 9 additions and 30 deletions.
3 changes: 1 addition & 2 deletions src/ecMatching.ml
Original file line number Diff line number Diff line change
Expand Up @@ -405,8 +405,7 @@ let f_match_core opts hyps (ue, ev) f1 f2 =

let var_form_match ((x, xty) : ident * ty) (f : form) =
match EV.get x !ev.evm_form with
| None ->
failure ()
| None -> assert false

| Some `Unset ->
let f = norm f in
Expand Down
36 changes: 8 additions & 28 deletions tests/split.ec
Original file line number Diff line number Diff line change
Expand Up @@ -3,33 +3,13 @@ require import AllCore.

print andWr.

lemma test : forall a b c d e f, a && b /\ c && d /\ e /\ f.
lemma test : forall a b c d e f,
a && b /\ c && d =>
e /\ f =>
a && b /\ c && d /\ e /\ f.
proof.
move=> *.

split 5.
split.
admit.



gl = a && b
gr = c /\ d

proja2 gl = b

conja (proja1 gl) (conj (proja2 gl) gr) = a && (b /\ (c /\ d))



admit.



admit.




abort.

split 3.
assumption.
assumption.
qed.

0 comments on commit 99ff0ce

Please sign in to comment.