comparison src/Predicates.v @ 205:f05514cc6c0d

'make doc' works with 8.2
author Adam Chlipala <adamc@hcoop.net>
date Fri, 06 Nov 2009 12:15:05 -0500
parents 71ade09024ac
children 90af611e2993
comparison
equal deleted inserted replaced
204:cbf2f74a5130 205:f05514cc6c0d
71 71
72 Print False. 72 Print False.
73 (** [[ 73 (** [[
74 74
75 Inductive False : Prop := 75 Inductive False : Prop :=
76
76 ]] *) 77 ]] *)
77 78
78 (** We can conclude anything from [False], doing case analysis on a proof of [False] in the same way we might do case analysis on, say, a natural number. Since there are no cases to consider, any such case analysis succeeds immediately in proving the goal. *) 79 (** We can conclude anything from [False], doing case analysis on a proof of [False] in the same way we might do case analysis on, say, a natural number. Since there are no cases to consider, any such case analysis succeeds immediately in proving the goal. *)
79 80
80 Theorem False_imp : False -> 2 + 2 = 5. 81 Theorem False_imp : False -> 2 + 2 = 5.