From b9c06ced8e899854d06314b52d0182e123775afc Mon Sep 17 00:00:00 2001 From: Stefan Monnier Date: Fri, 6 Jun 2014 17:23:03 +0000 Subject: * coq/coq-smie.el: Fix precedence of 'else'. --- coq/ex/indent.v | 6 ++++++ 1 file changed, 6 insertions(+) (limited to 'coq/ex') diff --git a/coq/ex/indent.v b/coq/ex/indent.v index c452cd1b..7218fa63 100644 --- a/coq/ex/indent.v +++ b/coq/ex/indent.v @@ -40,6 +40,12 @@ Proof. }} Qed. +Let x (* Precedence of "else" w.r.t "," and "->"! *) + : if true then nat * nat else nat -> + nat + := (if true then 1 else 2, + 3). + Module Y. Lemma L : forall x:nat , nat_iter x (A:=nat) (plus 2) 0 >= x. Proof with auto with arith. -- cgit v1.2.3