diff options
author | Matthieu Sozeau <matthieu.sozeau@inria.fr> | 2015-09-23 14:10:03 +0200 |
---|---|---|
committer | Matthieu Sozeau <mattam@mattam.org> | 2015-10-02 15:54:10 +0200 |
commit | ff4d0d98ab0e0e81bd1acf9a7bf4b64913834911 (patch) | |
tree | 19f50acc2a294e79e86381d6e507b23c42dcf08c /theories | |
parent | 0d923ee82bfed8d33d677dafb4b8defa18e4fdd1 (diff) |
Remove Print Universe directive.
Diffstat (limited to 'theories')
-rw-r--r-- | theories/Init/Logic.v | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v index 375495c88..50f853f0e 100644 --- a/theories/Init/Logic.v +++ b/theories/Init/Logic.v @@ -370,7 +370,7 @@ Module EqNotations. End EqNotations. Import EqNotations. -Set Printing Universes. + Lemma rew_opp_r : forall A (P:A->Type) (x y:A) (H:x=y) (a:P y), rew H in rew <- H in a = a. Proof. intros. |