Skip to content
Snippets Groups Projects
Commit c2c98f80 authored by Ralf Jung's avatar Ralf Jung
Browse files

reduce TC assumptions made by fin_to_set

parent 1422f908
No related branches found
No related tags found
No related merge requests found
...@@ -875,7 +875,7 @@ Section option_and_list_to_set. ...@@ -875,7 +875,7 @@ Section option_and_list_to_set.
End option_and_list_to_set. End option_and_list_to_set.
(** * Finite types to sets. *) (** * Finite types to sets. *)
Definition fin_to_set (A : Type) `{SemiSet A C, Finite A} : C := Definition fin_to_set (A : Type) `{Singleton A C, Empty C, Union C, Finite A} : C :=
list_to_set (enum A). list_to_set (enum A).
Section fin_to_set. Section fin_to_set.
...@@ -890,7 +890,6 @@ Section fin_to_set. ...@@ -890,7 +890,6 @@ Section fin_to_set.
Proof. constructor. split; auto using elem_of_fin_to_set. Qed. Proof. constructor. split; auto using elem_of_fin_to_set. Qed.
End fin_to_set. End fin_to_set.
(** * Guard *) (** * Guard *)
Global Instance set_guard `{MonadSet M} : MGuard M := Global Instance set_guard `{MonadSet M} : MGuard M :=
λ P dec A x, match dec with left H => x H | _ => end. λ P dec A x, match dec with left H => x H | _ => end.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment