(************************************************************************) (* * The Coq Proof Assistant / The Coq Development Team *) (* v * Copyright INRIA, CNRS and contributors *) (* Squash A. Arguments squash {_} _. Inductive sEmpty : SProp :=. Inductive sUnit : SProp := stt. Set Primitive Projections. Record Ssig {A:Type} (P:A->SProp) := Sexists { Spr1 : A; Spr2 : P Spr1 }. Arguments Sexists {_} _ _ _. Arguments Spr1 {_ _} _. Arguments Spr2 {_ _} _. Lemma Spr1_inj {A P} {a b : @Ssig A P} (e : Spr1 a = Spr1 b) : a = b. Proof. destruct a,b;simpl in e. destruct e. reflexivity. Defined.