Skip to content
Snippets Groups Projects
Commit 92e7ad56 authored by Robbert Krebbers's avatar Robbert Krebbers
Browse files

Merge branch 'simpl-never-fix' into 'master'

Avoid relying on buggy simpl never behavior

See merge request !228
parents 7309dfa2 bfca791e
No related branches found
No related tags found
1 merge request!228Avoid relying on buggy simpl never behavior
Pipeline #41808 passed
...@@ -64,8 +64,8 @@ Lemma find_is_Some `{finA: Finite A} P `{∀ x, Decision (P x)} (x : A) : ...@@ -64,8 +64,8 @@ Lemma find_is_Some `{finA: Finite A} P `{∀ x, Decision (P x)} (x : A) :
Proof. Proof.
destruct finA as [xs Hxs HA]; unfold find, decode; simpl. destruct finA as [xs Hxs HA]; unfold find, decode; simpl.
intros Hx. destruct (list_find_elem_of P xs x) as [[i y] Hi]; auto. intros Hx. destruct (list_find_elem_of P xs x) as [[i y] Hi]; auto.
rewrite Hi; simpl. rewrite !Nat2Pos.id by done. simpl. rewrite Hi; unfold decode_nat, decode; simpl. rewrite !Nat2Pos.id by done.
apply list_find_Some in Hi; naive_solver. simpl. apply list_find_Some in Hi; naive_solver.
Qed. Qed.
Definition encode_fin `{Finite A} (x : A) : fin (card A) := Definition encode_fin `{Finite A} (x : A) : fin (card A) :=
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Please register or to comment