aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Factorial.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Arith/Factorial.v')
-rw-r--r--theories/Arith/Factorial.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/theories/Arith/Factorial.v b/theories/Arith/Factorial.v
index 71cef55ce..ca176a6c6 100644
--- a/theories/Arith/Factorial.v
+++ b/theories/Arith/Factorial.v
@@ -22,6 +22,8 @@ Fixpoint fact [n:nat]:nat:=
|(S n) => (mult (S n) (fact n))
end.
+Arguments Scope fact [ nat_scope ].
+
Lemma lt_O_fact : (n:nat)(lt O (fact n)).
Proof.
Induction n; Unfold lt; Simpl; Auto with arith.