blob: fdd609f5b2e73ced217957ddcc805bd421bf3172 (
plain)
1
2
3
4
5
6
7
8
9
|
Inductive sig2 (A : Type) (P Q : A -> Prop) : Type :=
exist2 : forall x : A, P x -> Q x -> {x : A | P x & Q x}.
Arguments sig2 [A]%type_scope (_ _)%type_scope
Arguments exist2 [A]%type_scope (_ _)%function_scope _ _ _
exists x : nat, x = x
: Prop
fun b : bool => if b then b else b
: bool -> bool
|